]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/relocation/ldrop_leq.ma
- partial commit: just the components below "computation"
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / relocation / ldrop_leq.ma
index cdca16bb53752e580a76306d00cb711455167075..91b20e72029387b813b2bd7d4c04553def7c5d5a 100644 (file)
@@ -59,6 +59,17 @@ elim (leq_ldrop_trans_be … (leq_sym … HL12) … HLK1) // -L1 -Hdi -Hide
 /3 width=3 by leq_sym, ex2_intro/
 qed-.
 
+lemma ldrop_O1_ex: ∀K2,i,L1. |L1| = |K2| + i →
+                   ∃∃L2. L1 ≃[0, i] L2 & ⇩[i] L2 ≡ K2.
+#K2 #i @(nat_ind_plus … i) -i
+[ /3 width=3 by leq_O2, ex2_intro/
+| #i #IHi #Y #Hi elim (ldrop_O1_lt Y 0) //
+  #I #L1 #V #H lapply (ldrop_inv_O2 … H) -H #H destruct
+  normalize in Hi; elim (IHi L1) -IHi
+  /3 width=5 by ldrop_drop, leq_pair, injective_plus_l, ex2_intro/
+]
+qed-.
+
 lemma dedropable_sn_TC: ∀R. dedropable_sn R → dedropable_sn (TC … R).
 #R #HR #L1 #K1 #s #d #e #HLK1 #K2 #H elim H -K2
 [ #K2 #HK12 elim (HR … HLK1 … HK12) -HR -K1
@@ -70,7 +81,7 @@ qed-.
 
 (* Inversion lemmas on equivalence ******************************************)
 
-lemma ldrop_O_inj: ∀i,L1,L2,K. ⇩[i] L1 ≡ K → ⇩[i] L2 ≡ K → L1 ≃[i, ∞] L2.
+lemma ldrop_O1_inj: ∀i,L1,L2,K. ⇩[i] L1 ≡ K → ⇩[i] L2 ≡ K → L1 ≃[i, ∞] L2.
 #i @(nat_ind_plus … i) -i
 [ #L1 #L2 #K #H <(ldrop_inv_O2 … H) -K #H <(ldrop_inv_O2 … H) -L1 //
 | #i #IHi * [2: #L1 #I1 #V1 ] * [2,4: #L2 #I2 #V2 ] #K #HLK1 #HLK2 //