]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/static_2/static/lsubr.ma
update in ground_2, static_2, basic_2
[helm.git] / matita / matita / contribs / lambdadelta / static_2 / static / lsubr.ma
index 5ff763dcbe66125b8476a457ce297d4c059cac00..a6197c52f335d2de225073899508cfc74aa0c1ef 100644 (file)
 (*                                                                        *)
 (**************************************************************************)
 
+include "ground_2/xoa/ex_2_3.ma".
+include "ground_2/xoa/ex_3_2.ma".
+include "ground_2/xoa/ex_3_3.ma".
+include "ground_2/xoa/ex_3_4.ma".
 include "static_2/notation/relations/lrsubeqc_2.ma".
 include "static_2/syntax/lenv.ma".
 
@@ -42,7 +46,7 @@ fact lsubr_inv_atom1_aux: ∀L1,L2. L1 ⫃ L2 → L1 = ⋆ → L2 = ⋆.
 #L1 #L2 * -L1 -L2 //
 [ #I #L1 #L2 #_ #H destruct
 | #L1 #L2 #V #W #_ #H destruct
-| #I1 #I2 #L1 #L2 #V #_ #H destruct  
+| #I1 #I2 #L1 #L2 #V #_ #H destruct
 ]
 qed-.
 
@@ -108,7 +112,7 @@ lemma lsubr_inv_abst1:
       ∨∨ ∃∃K2. K1 ⫃ K2 & L2 = K2.ⓛW
        | ∃∃I2,K2. K1 ⫃ K2 & L2 = K2.ⓤ{I2}.
 #K1 #L2 #W #H elim (lsubr_inv_bind1 … H) -H *
-/3 width=4 by ex2_2_intro, ex2_intro, or_introl, or_intror/ 
+/3 width=4 by ex2_2_intro, ex2_intro, or_introl, or_intror/
 #K2 #V2 #W2 #_ #_ #H destruct
 qed-.
 
@@ -129,7 +133,7 @@ lemma lsubr_inv_pair2:
 #I #L1 #K2 #W #H elim (lsubr_inv_bind2 … H) -H *
 [ /3 width=3 by ex2_intro, or_introl/
 | #K1 #X #V #HK12 #H1 #H2 destruct /3 width=4 by ex3_2_intro, or_intror/
-| #J1 #J1 #K1 #V #_ #_ #H destruct   
+| #J1 #J1 #K1 #V #_ #_ #H destruct
 ]
 qed-.