]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/reducibility/cfpr_cpr.ma
update in basic_2
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / reducibility / cfpr_cpr.ma
index a46c9776bc2cf315c47e8342907a149633cf78ba..a1e20a025ef1766958ce7bbaa8cfde76b5327e4b 100644 (file)
@@ -12,7 +12,6 @@
 (*                                                                        *)
 (**************************************************************************)
 
-include "basic_2/unfold/ltpss_sn_alt.ma".
 include "basic_2/reducibility/cpr_tpss.ma".
 include "basic_2/reducibility/cpr_cpr.ma".
 include "basic_2/reducibility/cfpr_ltpss.ma".
@@ -30,7 +29,7 @@ lemma fpr_all: ∀L1,L. L1 ➡ L → ∀L2,T1,T2. L ⊢ T1 ➡ T2 →
 | #I #L1 #L #V1 #V #_ #HV1 #IH #X #T1 #T2 #HT12 #H
   elim (ltpss_sn_inv_tpss21 … H ?) -H // <minus_plus_m_m #L2 #V2 #HL2 #HV2 #H destruct
   lapply (cpr_bind_dx false … HV1 HT12) -HV1 -HT12 #HT12
-  lapply (cpr_tpss_trans … HT12 (-ⓑ{I}V2.T2) ?) -HT12 /2 width=1/ -HV2 /3 width=1/
+  lapply (cpr_tpss_trans … HT12 (-ⓑ{I}V2.T2) 0 (|L|) ?) -HT12 /2 width=1/ -HV2 /3 width=1/
 ]
 qed.
 
@@ -50,7 +49,7 @@ lemma cfpr_inv_all: ∀L1,L2,L0,T1,T2. L0 ⊢ ⦃L1, T1⦄ ➡ ⦃L2, T2⦄ →
   elim (append_inj_dx … H ?) -H // -HX #_ #H destruct -X
   lapply (ltpss_sn_fwd_length … HL2) >append_length >append_length #H
   lapply (injective_plus_r … H) -H #H
-  @(ex3_1_intro … (⋆.ⓑ{I}V@@Y)) <append_assoc // -HT12
+  @(ex3_intro … (⋆.ⓑ{I}V@@Y)) <append_assoc // -HT12
   <append_assoc [ /3 width=1/ ] -HV1 -HY
   >append_length <associative_plus
   @(ltpss_sn_dx_trans_eq … HL2) -HL2 >H -H >commutative_plus /3 width=1/