X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fbasic_2%2Fetc%2Fllpx_sn_alt2.etc;h=5a87c0da3cd6fb347fc2874ab76ebe5ed73f332e;hb=3325b784763ae9e6bac4307463071bb38e5641c9;hp=888f83ef4cb50eaad1bd5d2754d75235f7d7f73f;hpb=a0d25627e80a3a2fe68da954b68f6d541c6dbc34;p=helm.git diff --git a/matita/matita/contribs/lambdadelta/basic_2/etc/llpx_sn_alt2.etc b/matita/matita/contribs/lambdadelta/basic_2/etc/llpx_sn_alt2.etc index 888f83ef4..5a87c0da3 100644 --- a/matita/matita/contribs/lambdadelta/basic_2/etc/llpx_sn_alt2.etc +++ b/matita/matita/contribs/lambdadelta/basic_2/etc/llpx_sn_alt2.etc @@ -15,104 +15,6 @@ include "basic_2/substitution/cofrees_lift.ma". include "basic_2/substitution/llpx_sn_alt1.ma". -lemma le_plus_xSy_O_false: ∀x,y. x + S y ≤ 0 → ⊥. -#x #y #H lapply (le_n_O_to_eq … H) -H minus_plus_plus_l - #Hd #He lapply (le_plus_to_le_r … Hd) -Hd - #Hd >IHL12 // -L2 >plus_minus /2 width=3 by transitive_le/ -] -qed-. - -lemma ldrop_fwd_length_le_ge: ∀L1,L2,d,e,s. ⇩[s, d, e] L1 ≡ L2 → d ≤ |L1| → |L1| - d ≤ e → |L2| = d. -#L1 #L2 #d #e #s #H elim H -L1 -L2 -d -e normalize -[ /2 width=1 by le_n_O_to_eq/ -| #I #L #V #_ minus_plus_plus_l - #L #HL1 #HL2 elim (lt_or_ge (|L1|) (e2-e1)) #H0 - [ elim (ldrop_inv_O1_gt … HL1 H0) -HL1 #H1 #H2 destruct - elim (ldrop_inv_atom1 … HL2) -HL2 #H #_ destruct - @(ex2_intro … (⋆)) [ @ldrop_O1_ge normalize // ] - @ldrop_atom #H destruct - | elim (ldrop_O1_pair … HL1 H0 I V) -HL1 -H0 /3 width=5 by ldrop_drop, ex2_intro/ - ] - ] -| #I #L1 #L2 #V1 #V2 #d #e2 #_ #HV21 #IHL12 #e1 #He12 elim (IHL12 … He12) -IHL12 - #L #HL1 #HL2 elim (lift_split … HV21 d e1) -HV21 /3 width=5 by ldrop_skip, ex2_intro/ -] -qed-. - (* LAZY SN POINTWISE EXTENSION OF A CONTEXT-SENSITIVE REALTION FOR TERMS ****) (* alternative definition of llpx_sn (not recursive) *)