X-Git-Url: http://git.megacz.com/?a=blobdiff_plain;f=src%2FNaturalDeduction.v;h=407948b134bc763b3cad1963a8ce341bc5df117d;hb=0aa54e44e3ecbc2ad27ce793ea66ce6aad132776;hp=f8baff0a4051152da2b85477f06a80bbb9ac65b0;hpb=ee7da23597402df671f18320edff6604f5f6de7c;p=coq-hetmet.git diff --git a/src/NaturalDeduction.v b/src/NaturalDeduction.v index f8baff0..407948b 100644 --- a/src/NaturalDeduction.v +++ b/src/NaturalDeduction.v @@ -1,5 +1,8 @@ (*********************************************************************************************************************************) -(* NaturalDeduction: structurally explicit proofs in Coq *) +(* NaturalDeduction: *) +(* *) +(* Structurally explicit natural deduction proofs. *) +(* *) (*********************************************************************************************************************************) Generalizable All Variables. @@ -299,6 +302,14 @@ Section Natural_Deduction. apply q2. subst. apply cnd0. Defined. + (* undo the above *) + Fixpoint closedNDtoNormalND {c}(cnd:ClosedND c) : ND [] c := + match cnd in ClosedND C return ND [] C with + | cnd_weak => nd_id0 + | cnd_rule h c cndh rhc => closedNDtoNormalND cndh ;; nd_rule rhc + | cnd_branch c1 c2 cnd1 cnd2 => nd_llecnac ;; nd_prod (closedNDtoNormalND cnd1) (closedNDtoNormalND cnd2) + end. + Close Scope nd_scope. Open Scope pf_scope.