src/ZF/Induct/Binary_Trees.thy
changeset 46900 73555abfa267
parent 46822 95f1e700b712
child 58871 c399ae4b836f
--- a/src/ZF/Induct/Binary_Trees.thy	Tue Mar 13 14:17:42 2012 +0100
+++ b/src/ZF/Induct/Binary_Trees.thy	Tue Mar 13 14:44:16 2012 +0100
@@ -123,10 +123,10 @@
 *}
 
 lemma n_leaves_reflect: "t \<in> bt(A) ==> n_leaves(bt_reflect(t)) = n_leaves(t)"
-  by (induct set: bt) (simp_all add: add_commute n_leaves_type)
+  by (induct set: bt) (simp_all add: add_commute)
 
 lemma n_leaves_nodes: "t \<in> bt(A) ==> n_leaves(t) = succ(n_nodes(t))"
-  by (induct set: bt) (simp_all add: add_succ_right)
+  by (induct set: bt) simp_all
 
 text {*
   Theorems about @{term bt_reflect}.