X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fbasic_2%2Frelocation%2Flexs.ma;h=b002e073af1af7be489b4f845d88376be49088cf;hb=632c54beaf67e68a1eeeec22274466157003b779;hp=4e0c82132f46da99512e1eddbba8a149709d98d7;hpb=b4b5f03ffca4f250a1dc02f277b70e4f33ac8a9b;p=helm.git diff --git a/matita/matita/contribs/lambdadelta/basic_2/relocation/lexs.ma b/matita/matita/contribs/lambdadelta/basic_2/relocation/lexs.ma index 4e0c82132..b002e073a 100644 --- a/matita/matita/contribs/lambdadelta/basic_2/relocation/lexs.ma +++ b/matita/matita/contribs/lambdadelta/basic_2/relocation/lexs.ma @@ -206,6 +206,17 @@ lemma lexs_co: ∀RN1,RP1,RN2,RP2. /3 width=1 by lexs_atom, lexs_next, lexs_push/ qed-. +lemma lexs_co_isid: ∀RN1,RP1,RN2,RP2. + (∀L1,T1,T2. RP1 L1 T1 T2 → RP2 L1 T1 T2) → + ∀f,L1,L2. L1 ⦻*[RN1, RP1, f] L2 → 𝐈⦃f⦄ → + L1 ⦻*[RN2, RP2, f] L2. +#RN1 #RP1 #RN2 #RP2 #HR #f #L1 #L2 #H elim H -f -L1 -L2 // +#f #I #K1 #K2 #V1 #V2 #_ #HV12 #IH #H +[ elim (isid_inv_next … H) -H // +| /4 width=3 by lexs_push, isid_inv_push/ +] +qed-. + lemma sle_lexs_trans: ∀RN,RP. (∀L,T1,T2. RN L T1 T2 → RP L T1 T2) → ∀f2,L1,L2. L1 ⦻*[RN, RP, f2] L2 → ∀f1. f1 ⊆ f2 → L1 ⦻*[RN, RP, f1] L2. @@ -231,3 +242,16 @@ lemma sle_lexs_conf: ∀RN,RP. (∀L,T1,T2. RP L T1 T2 → RN L T1 T2) → #g2 #H #H2 destruct /3 width=5 by lexs_next/ ] qed-. + +lemma lexs_sle_split: ∀R1,R2,RP. (∀L. reflexive … (R1 L)) → (∀L. reflexive … (R2 L)) → + ∀f,L1,L2. L1 ⦻*[R1, RP, f] L2 → ∀g. f ⊆ g → + ∃∃L. L1 ⦻*[R1, RP, g] L & L ⦻*[R2, cfull, f] L2. +#R1 #R2 #RP #HR1 #HR2 #f #L1 #L2 #H elim H -f -L1 -L2 +[ /2 width=3 by lexs_atom, ex2_intro/ ] +#f #I #L1 #L2 #V1 #V2 #_ #HV12 #IH #y #H +[ elim (sle_inv_nx … H ??) -H [ |*: // ] #g #Hfg #H destruct + elim (IH … Hfg) -IH -Hfg /3 width=5 by lexs_next, ex2_intro/ +| elim (sle_inv_px … H ??) -H [1,3: * |*: // ] #g #Hfg #H destruct + elim (IH … Hfg) -IH -Hfg /3 width=5 by lexs_next, lexs_push, ex2_intro/ +] +qed-.