]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/computation/cpxs_tstc.ma
update in ground_2 and basic_2 ...
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / computation / cpxs_tstc.ma
index ec36d47f1432e71b0685fbf8d2607ed5e4b7cf60..c0a202ae5db8fd6b56f6b89d86e555bcc8a08566 100644 (file)
@@ -19,7 +19,7 @@ include "basic_2/computation/lpxs_cpxs.ma".
 
 (* Forward lemmas involving same top term constructor ***********************)
 
-lemma cpxs_fwd_cnx: ∀h,g,G,L,T. ⦃G, L⦄ ⊢ 𝐍[h, g]⦃T⦄ → ∀U. ⦃G, L⦄ ⊢ T ➡*[h, g] U → T ≃ U.
+lemma cpxs_fwd_cnx: ∀h,g,G,L,T. ⦃G, L⦄ ⊢ ➡[h, g] 𝐍⦃T⦄ → ∀U. ⦃G, L⦄ ⊢ T ➡*[h, g] U → T ≃ U.
 #h #g #G #L #T #HT #U #H
 >(cpxs_inv_cnx1 … H HT) -G -L -T //
 qed-.
@@ -34,7 +34,7 @@ elim (cpxs_inv_sort1 … H) -H #n #l generalize in match k; -k @(nat_ind_plus 
   elim (IHn … Hnl) -IHn
   [ #H lapply (tstc_inv_atom1 … H) -H #H >H -H /2 width=1 by or_intror/
   | generalize in match Hnl; -Hnl @(nat_ind_plus … n) -n
-    /4 width=3 by cpxs_strap2, cpx_sort, or_intror/
+    /4 width=3 by cpxs_strap2, cpx_st, or_intror/
   | >iter_SO >iter_n_Sm //
   ]
 ]