X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambda_delta%2Fbasic_2%2Freducibility%2Flfpr_cpr.ma;fp=matita%2Fmatita%2Fcontribs%2Flambda_delta%2Fbasic_2%2Freducibility%2Flfpr_cpr.ma;h=0000000000000000000000000000000000000000;hb=e8998d29ab83e7b6aa495a079193705b2f6743d3;hp=2a40f58bd2c83ddd6b094bc1e1a13156de9e5c38;hpb=bde429ac54e48de74b3d8b1df72dfcb86aa9bae5;p=helm.git diff --git a/matita/matita/contribs/lambda_delta/basic_2/reducibility/lfpr_cpr.ma b/matita/matita/contribs/lambda_delta/basic_2/reducibility/lfpr_cpr.ma deleted file mode 100644 index 2a40f58bd..000000000 --- a/matita/matita/contribs/lambda_delta/basic_2/reducibility/lfpr_cpr.ma +++ /dev/null @@ -1,29 +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/unfold/ltpss_sn_ltpss_sn.ma". -include "basic_2/reducibility/cpr.ma". -include "basic_2/reducibility/lfpr.ma". - -(* FOCALIZED PARALLEL REDUCTION FOR LOCAL ENVIRONMENTS **********************) - -(* Advanced properties ****************************************************) - -lemma lfpr_pair_cpr: ∀L1,L2. ⦃L1⦄ ➡ ⦃L2⦄ → ∀V1,V2. L2 ⊢ V1 ➡ V2 → - ∀I. ⦃L1. ⓑ{I} V1⦄ ➡ ⦃L2. ⓑ{I} V2⦄. -#L1 #L2 * #L #HL1 #HL2 #V1 #V2 * -<(ltpss_sn_fwd_length … HL2) #V #HV1 #HV2 #I -lapply (ltpss_sn_tpss_trans_eq … HV2 … HL2) -HV2 #V2 -@(ex2_1_intro … (L.ⓑ{I}V)) /2 width=1/ (**) (* explicit constructor *) -qed.