X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;ds=sidebyside;f=matita%2Fmatita%2Fcontribs%2Flambda_delta%2Fbasic_2%2Fetc%2Fcsup%2Fysteps_csups.etc;fp=matita%2Fmatita%2Fcontribs%2Flambda_delta%2Fbasic_2%2Fetc%2Fcsup%2Fysteps_csups.etc;h=2e48f396d1c023f6969cbd3b949449a3cd93d0b2;hb=53f874fba5b9c39a788085515a4fefe5d29281da;hp=0000000000000000000000000000000000000000;hpb=f7386d0b74f935f07ede4be46d0489a233d68b85;p=helm.git diff --git a/matita/matita/contribs/lambda_delta/basic_2/etc/csup/ysteps_csups.etc b/matita/matita/contribs/lambda_delta/basic_2/etc/csup/ysteps_csups.etc new file mode 100644 index 000000000..2e48f396d --- /dev/null +++ b/matita/matita/contribs/lambda_delta/basic_2/etc/csup/ysteps_csups.etc @@ -0,0 +1,28 @@ +(**************************************************************************) +(* ___ *) +(* ||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/computation/yprs_csups.ma". +include "basic_2/computation/ysteps.ma". + +(* ITERATED STEP OF HYPER PARALLEL COMPUTATION ON CLOSURES ******************) + +(* Properties on iterated supclosure ****************************************) + +lemma csups_ysteps: ∀h,g,L1,L2,T1,T2. ⦃L1, T1⦄ >* ⦃L2, T2⦄ → + h ⊢ ⦃L1, T1⦄ •⭃*[g] ⦃L2, T2⦄. +#h #g #L1 #L2 #T1 #T2 #H +lapply (csups_fwd_cw … H) #H1 +@ysteps_intro /2 width=1/ -H #H2 #H3 destruct +elim (lt_refl_false … H1) +qed.