]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/contribs/lambdadelta/basic_2/computation/fsb.ma
- "big tree" theorem is now proved up to some conjectures involving
[helm.git] / matita / matita / contribs / lambdadelta / basic_2 / computation / fsb.ma
index 64090eec97d6003aa5b9807f9164c43413019dfb..1616402dec981972dba696ee60e6fe0405a57dc0 100644 (file)
@@ -13,7 +13,7 @@
 (**************************************************************************)
 
 include "basic_2/notation/relations/btsn_5.ma".
-include "basic_2/computation/fpbc.ma".
+include "basic_2/computation/fpbu.ma".
 include "basic_2/computation/csx_alt.ma".
 
 (* "BIG TREE" STRONGLY NORMALIZING TERMS ************************************)
@@ -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_cprs, fpbc_cpxs/
+#h #g #G #L #T #H elim H -G -L -T /5 width=1 by csx_intro_cprs, fpbu_cpxs/
 qed-.