src/HOL/ex/BT.thy
changeset 8339 bcadeb9c7095
parent 5184 9b8547a9496a
child 11024 23bf8d787b04
--- a/src/HOL/ex/BT.thy	Sat Mar 04 11:42:12 2000 +0100
+++ b/src/HOL/ex/BT.thy	Sat Mar 04 11:52:42 2000 +0100
@@ -6,9 +6,10 @@
 Binary trees (based on the ZF version)
 *)
 
-BT = List +
+BT = Main +
 
-datatype 'a bt = Lf  |  Br 'a ('a bt) ('a bt)
+datatype 'a bt = Lf
+               | Br 'a ('a bt) ('a bt)
   
 consts
     n_nodes     :: 'a bt => nat