src/HOL/Library/Tree.thy
changeset 63829 6a05c8cbf7de
parent 63770 a67397b13eb5
child 63861 90360390a916
--- a/src/HOL/Library/Tree.thy	Fri Sep 09 13:39:21 2016 +0200
+++ b/src/HOL/Library/Tree.thy	Fri Sep 09 14:15:16 2016 +0200
@@ -230,7 +230,8 @@
 
 subsection \<open>Balanced\<close>
 
-abbreviation "balanced t \<equiv> (height t - min_height t \<le> 1)"
+definition balanced :: "'a tree \<Rightarrow> bool" where
+"balanced t = (height t - min_height t \<le> 1)"
 
 text\<open>Balanced trees have optimal height:\<close>
 
@@ -262,7 +263,7 @@
   hence *: "min_height t < height t'" by simp
   have "min_height t + 1 = height t"
     using min_hight_le_height[of t] assms(1) False
-    by (simp add: complete_iff_height)
+    by (simp add: complete_iff_height balanced_def)
   with * show ?thesis by arith
 qed