fixed the definition of "depth"
authorpaulson
Tue, 26 Sep 2006 11:11:57 +0200
changeset 20711 8b52cdaee86c
parent 20710 384bfce59254
child 20712 b3cd1233167f
fixed the definition of "depth"
src/HOL/ex/BT.thy
--- a/src/HOL/ex/BT.thy	Tue Sep 26 11:09:33 2006 +0200
+++ b/src/HOL/ex/BT.thy	Tue Sep 26 11:11:57 2006 +0200
@@ -3,7 +3,7 @@
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1995  University of Cambridge
 
-Binary trees (based on the ZF version).
+Binary trees
 *)
 
 header {* Binary trees *}
@@ -35,7 +35,7 @@
 
 primrec
   "depth Lf = 0"
-  "depth (Br a t1 t2) = max (depth t1) (depth t2)"
+  "depth (Br a t1 t2) = Suc (max (depth t1) (depth t2))"
 
 primrec
   "reflect Lf = Lf"
@@ -75,8 +75,8 @@
   done
 
 lemma depth_reflect: "depth (reflect t) = depth t"
-  apply (induct t)
-   apply (simp_all add: max_ac)
+  apply (induct t) 
+   apply auto
   done
 
 text {*