X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fbasic_2%2Fetc%2Fssta1%2Fcpes.etc;fp=matita%2Fmatita%2Fcontribs%2Flambdadelta%2Fbasic_2%2Fetc%2Fssta1%2Fcpes.etc;h=0000000000000000000000000000000000000000;hb=5d669f492522b055f76c627eb89da97d0be05c2a;hp=7aeb07cb07bb1c25afe1c637faaf250652004107;hpb=63c047cae0056da7a69cb0740336d12259fbeb1a;p=helm.git diff --git a/matita/matita/contribs/lambdadelta/basic_2/etc/ssta1/cpes.etc b/matita/matita/contribs/lambdadelta/basic_2/etc/ssta1/cpes.etc deleted file mode 100644 index 7aeb07cb0..000000000 --- a/matita/matita/contribs/lambdadelta/basic_2/etc/ssta1/cpes.etc +++ /dev/null @@ -1,46 +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/notation/relations/dpconvstar_6.ma". -include "basic_2/unfold/lsstas.ma". -include "basic_2/equivalence/cpcs.ma". - -(* DECOMPOSED EXTENDED PARALLEL EQUIVALENCE FOR TERMS ***********************) - -definition cpes: ∀h. sd h → relation4 genv lenv term term ≝ - λh,g,G,L,T1,T2. - ∃∃T,l1,l2. l2 ≤ l1 & ⦃G, L⦄ ⊢ T1 ▪[h, g] l1 & ⦃G, L⦄ ⊢ T1 •*[h, g, l2] T & ⦃G, L⦄ ⊢ T ⬌* T2. - -interpretation "decomposed extended parallel equivalence (term)" - 'DPConvStar h g G L T1 T2 = (cpes h g G L T1 T2). - -(* Basic properties *********************************************************) - -lemma ssta_cpcs_cpes: ∀h,g,G,L,T1,T,T2,l. ⦃G, L⦄ ⊢ T1 ▪[h, g] l+1 → ⦃G, L⦄ ⊢ T1 •[h, g] T → - ⦃G, L⦄ ⊢ T ⬌* T2 → ⦃G, L⦄ ⊢ T1 •*⬌*[h, g] T2. -/3 width=7/ qed. - -lemma lsstas_cpes: ∀h,g,G,L,T1,T2,l. ⦃G, L⦄ ⊢ T1 ▪[h, g] l → ⦃G, L⦄ ⊢ T1 •*[h, g, l] T2 → ⦃G, L⦄ ⊢ T1 •*⬌*[h, g] T2. -/2 width=7/ qed. - -lemma cpcs_cpes: ∀h,g,G,L,T1,T2,l. ⦃G, L⦄ ⊢ T1 ▪[h, g] l → ⦃G, L⦄ ⊢ T1 ⬌* T2 → ⦃G, L⦄ ⊢ T1 •*⬌*[h, g] T2. -/2 width=7/ qed. - -lemma cpes_refl: ∀h,g,G,L,T,l. ⦃G, L⦄ ⊢ T ▪[h, g] l → ⦃G, L⦄ ⊢ T •*⬌*[h, g] T. -/2 width=2/ qed. - -lemma cpes_strap1: ∀h,g,G,L,T1,T,T2. - ⦃G, L⦄ ⊢ T1 •*⬌*[h, g] T → ⦃G, L⦄ ⊢ T ⬌ T2 → ⦃G, L⦄ ⊢ T1 •*⬌*[h, g] T2. -#h #g #G #L #T1 #T #T2 * /3 width=9/ -qed.