X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fground_2%2Frelocation%2Frtmap_sor.ma;h=bc2a7dda6efd52eb61c36537bf43a5fdf8484e59;hb=a78df6200d61b34a67cb1cba9edf984aae470530;hp=efa6b54d9d60f1078d6b26672fa5d1c9615ce17a;hpb=614542345e3e9c88722fdbc32c24a14b9a6c71d1;p=helm.git diff --git a/matita/matita/contribs/lambdadelta/ground_2/relocation/rtmap_sor.ma b/matita/matita/contribs/lambdadelta/ground_2/relocation/rtmap_sor.ma index efa6b54d9..bc2a7dda6 100644 --- a/matita/matita/contribs/lambdadelta/ground_2/relocation/rtmap_sor.ma +++ b/matita/matita/contribs/lambdadelta/ground_2/relocation/rtmap_sor.ma @@ -323,6 +323,18 @@ qed. lemma sor_isid: ∀f1,f2,f. 𝐈⦃f1⦄ → 𝐈⦃f2⦄ → 𝐈⦃f⦄ → f1 ⋓ f2 ≡ f. /4 width=3 by sor_eq_repl_back2, sor_eq_repl_back1, isid_inv_eq_repl/ qed. +(* Inversion lemmas with tail ***********************************************) + +lemma sor_inv_tl_sn: ∀f1,f2,f. ⫱f1 ⋓ f2 ≡ f → f1 ⋓ ⫯f2 ≡ ⫯f. +#f1 #f2 #f elim (pn_split f1) * +#g1 #H destruct /2 width=7 by sor_pn, sor_nn/ +qed-. + +lemma sor_inv_tl_dx: ∀f1,f2,f. f1 ⋓ ⫱f2 ≡ f → ⫯f1 ⋓ f2 ≡ ⫯f. +#f1 #f2 #f elim (pn_split f2) * +#g2 #H destruct /2 width=7 by sor_np, sor_nn/ +qed-. + (* Inversion lemmas with test for identity **********************************) lemma sor_isid_inv_sn: ∀f1,f2,f. f1 ⋓ f2 ≡ f → 𝐈⦃f1⦄ → f2 ≗ f.