X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fbasic_2A%2Fetc%2Ffsup%2Fldrop_fsups.etc;fp=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fbasic_2A%2Fetc%2Ffsup%2Fldrop_fsups.etc;h=dc4d7e9f4b6356b73e48030475ba2ad01eab1577;hb=1fd63df4c77f5c24024769432ea8492748b4ac79;hp=0000000000000000000000000000000000000000;hpb=277fc8ff21ce3dbd6893b1994c55cf5c06a98355;p=helm.git diff --git a/matita/matita/contribs/lambdadelta/basic_2A/etc/fsup/ldrop_fsups.etc b/matita/matita/contribs/lambdadelta/basic_2A/etc/fsup/ldrop_fsups.etc new file mode 100644 index 000000000..dc4d7e9f4 --- /dev/null +++ b/matita/matita/contribs/lambdadelta/basic_2A/etc/fsup/ldrop_fsups.etc @@ -0,0 +1,30 @@ +(**************************************************************************) +(* ___ *) +(* ||M|| *) +(* ||A|| A project by Andrea Asperti *) +(* ||T|| *) +(* ||I|| Developers: *) +(* ||T|| The HELM team. *) +(* ||A|| http://helm.cs.unibo.it *) +(* \ / *) +(* \ / This file is distributed under the terms of the *) +(* v GNU General Public License Version 2 *) +(* *) +(**************************************************************************) + +include "basic_2/grammar/fsups.ma". +include "basic_2/substitution/ldrop_fsup.ma". + +(* LOCAL ENVIRONMENT SLICING ************************************************) + +(* Inversion lemmas on plus-iterated supclosure ****************************) + +lemma fsupp_inv_atom1_fsups: ∀J,L1,L2,T2. ⦃L1, ⓪{J}⦄ ⊃+ ⦃L2, T2⦄ → + ∃∃I,K,V,i. ⇩[0, i] L1 ≡ K.ⓑ{I}V & + ⦃K, V⦄ ⊃* ⦃L2, T2⦄ & J = LRef i. +#J #L1 #L2 #T2 #H @(fsupp_ind … H) -L2 -T2 +[ #L2 #T2 #H + elim (fsup_inv_atom1_ldrop … H) -H * #i #HL12 #H destruct /2 width=7/ +| #L #T #L2 #T2 #_ #HT2 * #I #K #V #i #HLK #HVT #H destruct /3 width=8/ +] +qed-.