src/HOL/Data_Structures/Balance.thy
changeset 64540 f1f4ba6d02c9
parent 64533 172f3a047f4a
child 64541 3d4331b65861
--- a/src/HOL/Data_Structures/Balance.thy	Sun Dec 04 21:40:50 2016 +0100
+++ b/src/HOL/Data_Structures/Balance.thy	Mon Dec 05 18:14:41 2016 +0100
@@ -26,7 +26,7 @@
 next
   assume *: "\<not> complete t"
   hence "height t = min_height t + 1"
-    using assms min_hight_le_height[of t]
+    using assms min_height_le_height[of t]
     by(auto simp add: balanced_def complete_iff_height)
   hence "2 ^ min_height t \<le> size1 t \<and> size1 t < 2 ^ (min_height t + 1)"
     by (metis * min_height_size1 size1_height_if_incomplete)
@@ -53,7 +53,7 @@
 next
   assume *: "\<not> complete t"
   hence **: "height t = min_height t + 1"
-    using assms min_hight_le_height[of t]
+    using assms min_height_le_height[of t]
     by(auto simp add: balanced_def complete_iff_height)
   hence 0: "2 ^ min_height t < size1 t \<and> size1 t \<le> 2 ^ (min_height t + 1)"
     by (metis "*" min_height_size1_if_incomplete size1_height)