]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/computation/csx_aaa.ma
some renaming and a minor addition
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / computation / csx_aaa.ma
index f1b70f0c73ad6a8f87b07cb81fbd45ace604cb31..6d8aa3ed940d1c521b036b99467f731f114b3c57 100644 (file)
@@ -12,9 +12,9 @@
 (*                                                                        *)
 (**************************************************************************)
 
-include "basic_2/computation/acp_aaa.ma".
+include "basic_2/computation/gcp_aaa.ma".
 include "basic_2/computation/cpxs_aaa.ma".
-include "basic_2/computation/csx_tstc_vector.ma".
+include "basic_2/computation/csx_tsts_vector.ma".
 
 (* CONTEXT-SENSITIVE EXTENDED STRONGLY NORMALIZING TERMS ********************)
 
@@ -22,7 +22,7 @@ include "basic_2/computation/csx_tstc_vector.ma".
 
 theorem aaa_csx: ∀h,g,G,L,T,A. ⦃G, L⦄ ⊢ T ⁝ A → ⦃G, L⦄ ⊢ ⬊*[h, g] T.
 #h #g #G #L #T #A #H
-@(acp_aaa … (csx_acp h g) (csx_acr h g) … H)
+@(gcr_aaa … (csx_gcp h g) (csx_gcr h g) … H)
 qed.
 
 (* Advanced eliminators *****************************************************)
@@ -32,7 +32,7 @@ fact aaa_ind_csx_aux: ∀h,g,G,L,A. ∀R:predicate term.
                             (∀T2. ⦃G, L⦄ ⊢ T1 ➡[h, g] T2 → (T1 = T2 → ⊥) → R T2) → R T1
                       ) →
                       ∀T. ⦃G, L⦄ ⊢ ⬊*[h, g] T → ⦃G, L⦄ ⊢ T ⁝ A → R T.
-#h #g #G #L #A #R #IH #T #H @(csx_ind … H) -T /4 width=5 by aaa_cpx_conf/
+#h #g #G #L #A #R #IH #T #H @(csx_ind … H) -T /4 width=5 by cpx_aaa_conf/
 qed-.
 
 lemma aaa_ind_csx: ∀h,g,G,L,A. ∀R:predicate term.
@@ -47,7 +47,7 @@ fact aaa_ind_csx_alt_aux: ∀h,g,G,L,A. ∀R:predicate term.
                                 (∀T2. ⦃G, L⦄ ⊢ T1 ➡*[h, g] T2 → (T1 = T2 → ⊥) → R T2) → R T1
                           ) →
                           ∀T. ⦃G, L⦄ ⊢ ⬊*[h, g] T → ⦃G, L⦄ ⊢ T ⁝ A → R T.
-#h #g #G #L #A #R #IH #T #H @(csx_ind_alt … H) -T /4 width=5 by aaa_cpxs_conf/
+#h #g #G #L #A #R #IH #T #H @(csx_ind_alt … H) -T /4 width=5 by cpxs_aaa_conf/
 qed-.
 
 lemma aaa_ind_csx_alt: ∀h,g,G,L,A. ∀R:predicate term.