X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fbasic_2A%2Fetc%2Fcny%2Flpxs_cpye.etc;fp=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fbasic_2A%2Fetc%2Fcny%2Flpxs_cpye.etc;h=a6f0f86bde726067b1903bb665cfe9c6259d456e;hb=1fd63df4c77f5c24024769432ea8492748b4ac79;hp=0000000000000000000000000000000000000000;hpb=277fc8ff21ce3dbd6893b1994c55cf5c06a98355;p=helm.git diff --git a/matita/matita/contribs/lambdadelta/basic_2A/etc/cny/lpxs_cpye.etc b/matita/matita/contribs/lambdadelta/basic_2A/etc/cny/lpxs_cpye.etc new file mode 100644 index 000000000..a6f0f86bd --- /dev/null +++ b/matita/matita/contribs/lambdadelta/basic_2A/etc/cny/lpxs_cpye.etc @@ -0,0 +1,36 @@ +(**************************************************************************) +(* ___ *) +(* ||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/substitution/cpye_lift.ma". +include "basic_2/reduction/lpx_cpye.ma". +include "basic_2/computation/cpxs_cpxs.ma". +include "basic_2/computation/lpxs.ma". + +(* SN EXTENDED PARALLEL COMPUTATION ON LOCAL ENVIRONMENTS *******************) + +(* Forward lemmas on evaluation for extended substitution *******************) + +lemma cpx_cpye_fwd_lpxs: ∀h,g,G,L1,L2. ⦃G, L1⦄ ⊢ ➡*[h, g] L2 → + ∀T1,T2. ⦃G, L1⦄ ⊢ T1 ➡[h, g] T2 → + ∀U1,d,e. ⦃G, L1⦄ ⊢ T1 ▶*[d, e] 𝐍⦃U1⦄ → + ∀U2. ⦃G, L2⦄ ⊢ T2 ▶*[d, e] 𝐍⦃U2⦄ → + ⦃G, L1⦄ ⊢ U1 ➡*[h, g] U2. +#h #g #G #L1 #L2 #H @(lpxs_ind_dx … H) -L1 +[ /3 width=9 by cpx_cpxs, cpx_cpye_fwd_lpx/ +| #L1 #L #HL1 #_ #IHL2 #T1 #T2 #HT12 #U1 #d #e #HTU1 #U2 #HTU2 + elim (cpye_total G L T2 d e) #X2 #HTX2 + lapply (cpx_cpye_fwd_lpx … HT12 … HL1 … HTU1 … HTX2) -T1 + /4 width=9 by lpx_cpxs_trans, cpxs_strap2/ (**) (* full auto too long: 41s *) +] +qed-.