tuned
authornipkow
Thu, 19 Jan 2017 12:39:46 +0100
changeset 64922 3fb4d7d00230
parent 64921 1cbfe46ad6b1
child 64923 7c340dcbc323
tuned
src/HOL/Library/Tree.thy
--- a/src/HOL/Library/Tree.thy	Wed Jan 18 21:03:39 2017 +0100
+++ b/src/HOL/Library/Tree.thy	Thu Jan 19 12:39:46 2017 +0100
@@ -147,7 +147,7 @@
     have "size1(Node l a r) = size1 l + size1 r" by simp
     also have "\<dots> \<le> 2 ^ height l + 2 ^ height r" using Node.IH by arith
     also have "\<dots> \<le> 2 ^ height r + 2 ^ height r" using True by simp
-    also have "\<dots> \<le> 2 ^ height (Node l a r)"
+    also have "\<dots> = 2 ^ height (Node l a r)"
       using True by (auto simp: max_def mult_2)
     finally show ?thesis .
   next