]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/computation/fsb.ma
- nnAuto: we catch TypeCheckerFailure generated at the end of
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / computation / fsb.ma
index a6d6627990518e5d4c17f1c964e643eb982bbc5f..4d44edb46b9e6469a747d7c4090d3d81b45edf49 100644 (file)
 (**************************************************************************)
 
 include "basic_2/notation/relations/btsn_5.ma".
-include "basic_2/reduction/fpbc.ma".
+include "basic_2/reduction/fpb.ma".
 include "basic_2/computation/csx.ma".
 
-(* "BIG TREE" STRONGLY NORMALIZING TERMS ************************************)
+(* "QRST" STRONGLY NORMALIZING TERMS ****************************************)
 
 inductive fsb (h) (g): relation3 genv lenv term ≝
 | fsb_intro: ∀G1,L1,T1. (
@@ -25,7 +25,7 @@ inductive fsb (h) (g): relation3 genv lenv term ≝
 .
 
 interpretation
-   "'big tree' strong normalization (closure)"
+   "'qrst' strong normalization (closure)"
    'BTSN h g G L T = (fsb h g G L T).
 
 (* Basic eliminators ********************************************************)
@@ -43,5 +43,5 @@ qed-.
 (* Basic inversion lemmas ***************************************************)
 
 lemma fsb_inv_csx: ∀h,g,G,L,T. ⦃G, L⦄ ⊢ ⦥[h, g] T → ⦃G, L⦄ ⊢ ⬊*[h, g] T.
-#h #g #G #L #T #H elim H -G -L -T /5 width=1 by csx_intro, fpbc_cpx/
+#h #g #G #L #T #H elim H -G -L -T /5 width=1 by csx_intro, fpb_cpx/
 qed-.