]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/reduction/cpx_cpys.ma
some notation renamed and fixed
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / reduction / cpx_cpys.ma
index 3c0507b32c9641b940d9638ca65e1e5bfe795316..6cb5a00ba9572ce0969b5ad993e9104ab2026896 100644 (file)
@@ -19,10 +19,10 @@ include "basic_2/reduction/cpx.ma".
 
 (* Properties on context-sensitive extended multiple substitution for terms *)
 
-lemma cpys_cpx: ∀h,g,G,L,T1,T2,d,e. ⦃G, L⦄ ⊢ T1 ▶*×[d, e] T2 → ⦃G, L⦄ ⊢ T1 ➡[h, g] T2.
+lemma cpys_cpx: ∀h,g,G,L,T1,T2,d,e. ⦃G, L⦄ ⊢ T1 ▶*[d, e] T2 → ⦃G, L⦄ ⊢ T1 ➡[h, g] T2.
 #h #g #G #L #T1 #T2 #d #e #H @(cpys_ind_alt … H) -G -L -T1 -T2 -d -e
 /2 width=7 by cpx_delta, cpx_bind, cpx_flat/
 qed.
 
-lemma cpy_cpx: ∀h,g,G,L,T1,T2,d,e. ⦃G, L⦄ ⊢ T1 ▶×[d, e] T2 → ⦃G, L⦄ ⊢ T1 ➡[h, g] T2.
+lemma cpy_cpx: ∀h,g,G,L,T1,T2,d,e. ⦃G, L⦄ ⊢ T1 ▶[d, e] T2 → ⦃G, L⦄ ⊢ T1 ➡[h, g] T2.
 /3 width=3 by cpy_cpys, cpys_cpx/ qed.