src/ZF/Induct/Tree_Forest.thy
changeset 41526 54b4686704af
parent 35762 af3ff2ba4c54
child 45602 2a858377c3d2
--- a/src/ZF/Induct/Tree_Forest.thy	Wed Jan 12 15:53:37 2011 +0100
+++ b/src/ZF/Induct/Tree_Forest.thy	Wed Jan 12 16:33:04 2011 +0100
@@ -176,7 +176,7 @@
   assumes "!!x. x \<in> A ==> h(x): B"
   shows map_tree_type: "t \<in> tree(A) ==> map(h,t) \<in> tree(B)"
     and map_forest_type: "f \<in> forest(A) ==> map(h,f) \<in> forest(B)"
-  using prems
+  using assms
   by (induct rule: tree'induct forest'induct) simp_all
 
 text {*