X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fbasic_2%2Freducibility%2Fxpr.ma;fp=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fbasic_2%2Freducibility%2Fxpr.ma;h=0000000000000000000000000000000000000000;hb=18bc3082b332504f60345245e716b62ae628e3a7;hp=7375349efe659651ab8659973413a664c43298a6;hpb=1ea0f459b4435459442c8afb113bae815e38986e;p=helm.git diff --git a/matita/matita/contribs/lambdadelta/basic_2/reducibility/xpr.ma b/matita/matita/contribs/lambdadelta/basic_2/reducibility/xpr.ma deleted file mode 100644 index 7375349ef..000000000 --- a/matita/matita/contribs/lambdadelta/basic_2/reducibility/xpr.ma +++ /dev/null @@ -1,32 +0,0 @@ -(**************************************************************************) -(* ___ *) -(* ||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/static/ssta.ma". -include "basic_2/reducibility/cpr.ma". - -(* EXTENDED PARALLEL REDUCTION ON TERMS *************************************) - -inductive xpr (h) (g) (L) (T1) (T2): Prop ≝ -| xpr_cpr : L ⊢ T1 ➡ T2 → xpr h g L T1 T2 -| xpr_ssta: ∀l. ⦃h, L⦄ ⊢ T1 •[g, l + 1] T2 → xpr h g L T1 T2 -. - -interpretation - "extended parallel reduction (term)" - 'XPRed h g L T1 T2 = (xpr h g L T1 T2). - -(* Basic properties *********************************************************) - -lemma xpr_refl: ∀h,g,L. reflexive … (xpr h g L). -/2 width=1/ qed.