Theory Natural_Deduction
theory Natural_Deduction
imports
Abstract_Completeness.Abstract_Completeness
Abstract_Rules
Entailment
begin
text ‹Our formalization of natural deduction builds on @{theory Abstract_Completeness.Abstract_Completeness} and refines and
concretizes the structure given there as follows
▪ The judgements are entailments consisting of a finite set of assumptions and a conclusion, which
are abstract formulas in the sense of @{theory Incredible_Proof_Machine.Abstract_Formula}.
▪ The abstract rules given in @{theory Incredible_Proof_Machine.Abstract_Rules} are used to decide the validity of a
step in the derivation.
›
text ‹A single setep in the derivation can either be the axiom rule, the cut rule, or one
of the given rules in @{theory Incredible_Proof_Machine.Abstract_Rules}.›