X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fbasic_2%2Fstatic%2Ffle_fle.ma;h=e756b43f773e1d873c3f67fc8a583d7f481abe65;hb=aff2f21cec89cf343297ae6bd720fc6573a3aba1;hp=77b284b11e288f1c8589a35ce444306d0e615868;hpb=6ed4f0127b8acb6caeba6fbfadef7f990dd7803e;p=helm.git diff --git a/matita/matita/contribs/lambdadelta/basic_2/static/fle_fle.ma b/matita/matita/contribs/lambdadelta/basic_2/static/fle_fle.ma index 77b284b11..e756b43f7 100644 --- a/matita/matita/contribs/lambdadelta/basic_2/static/fle_fle.ma +++ b/matita/matita/contribs/lambdadelta/basic_2/static/fle_fle.ma @@ -13,13 +13,62 @@ (**************************************************************************) include "basic_2/static/frees_frees.ma". -include "basic_2/static/fle.ma". +include "basic_2/static/fle_fqup.ma". (* FREE VARIABLES INCLUSION FOR RESTRICTED CLOSURES *************************) -(* Main properties **********************************************************) +(* Advanced inversion lemmas ************************************************) + +lemma fle_inv_voids_sn_frees_dx: ∀L1,L2,T1,T2,n. ⦃ⓧ*[n]L1, T1⦄ ⊆ ⦃L2, T2⦄ → + |L1| = |L2| → ∀f2. L2 ⊢ 𝐅*⦃T2⦄ ≡ f2 → + ∃∃f1. ⓧ*[n]L1 ⊢ 𝐅*⦃T1⦄ ≡ f1 & ⫱*[n]f1 ⊆ f2. +#L1 #L2 #T1 #T2 #n #H #HL12 #f2 #Hf2 +elim (fle_inv_voids_sn … H HL12) -H -HL12 #f1 #g2 #Hf1 #Hg2 #Hfg +lapply (frees_mono … Hg2 … Hf2) -Hg2 -Hf2 #Hfg2 +lapply (sle_eq_repl_back2 … Hfg … Hfg2) -g2 +/2 width=3 by ex2_intro/ +qed-. +(* Main properties **********************************************************) +(* theorem fle_trans: bi_transitive … fle. #L1 #L #T1 #T * #f1 #f #HT1 #HT #Hf1 #L2 #T2 * #g #f2 #Hg #HT2 #Hf2 /5 width=8 by frees_mono, sle_trans, sle_eq_repl_back2, ex3_2_intro/ qed-. +*) +theorem fle_bind_sn: ∀L1,L2,V1,T1,T. ⦃L1, V1⦄ ⊆ ⦃L2, T⦄ → ⦃L1.ⓧ, T1⦄ ⊆ ⦃L2, T⦄ → + ∀p,I. ⦃L1, ⓑ{p,I}V1.T1⦄ ⊆ ⦃L2, T⦄. +#L1 #L2 #V1 #T1 #T * -L1 #f1 #x #L1 #n1 #Hf1 #Hx #HL12 #Hf1x +>voids_succ #H #p #I +elim (fle_inv_voids_sn_frees_dx … H … Hx) -H // #f2 #Hf2 +