X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;ds=sidebyside;f=helm%2Fsoftware%2Fmatita%2Flibrary%2Fdemo%2Frealisability.ma;h=93b5e712f24724cee2d004ea2f30e65432e1f16b;hb=9eabe046c1182960de8cfdba96c5414224e3a61e;hp=0cd58c63dce78b1c70fe0640541c2d405c73621e;hpb=27bfea6a5157027d01f57b12ecacdd507b569864;p=helm.git diff --git a/helm/software/matita/library/demo/realisability.ma b/helm/software/matita/library/demo/realisability.ma index 0cd58c63d..93b5e712f 100644 --- a/helm/software/matita/library/demo/realisability.ma +++ b/helm/software/matita/library/demo/realisability.ma @@ -12,8 +12,6 @@ (* *) (**************************************************************************) -set "baseuri" "cic:/matita/demo/realisability/". - include "logic/connectives.ma". include "datatypes/constructors.ma". @@ -116,9 +114,8 @@ theorem correct: ∀F:SP.∀r:type_OF_SP F.modr F r → Prop_OF_SP F. | apply (proj2 ? ? H2) ] ] - | generalize in match H2; clear H2; - change in r with (type_OF_SP s + type_OF_SP s1); - elim r; simplify in H2; + | change in r with (type_OF_SP s + type_OF_SP s1); + elim r in H2 ⊢ %; simplify in H2; [ left; apply H; assumption | right; apply H1; assumption ] @@ -131,8 +128,7 @@ theorem correct: ∀F:SP.∀r:type_OF_SP F.modr F r → Prop_OF_SP F. | skip ] | simplify in r; - generalize in match H1; clear H1; - elim r; + elim r in H1 ⊢ %; apply (ex_intro ? ? a); apply H; assumption