src/HOL/ex/Tree23.thy
changeset 58249 180f1b3508ed
parent 55417 01fbfb60c33e
child 58310 91ea607a34d8
--- a/src/HOL/ex/Tree23.thy	Tue Sep 09 17:51:07 2014 +0200
+++ b/src/HOL/ex/Tree23.thy	Tue Sep 09 20:51:36 2014 +0200
@@ -21,16 +21,16 @@
 
 type_synonym key = int -- {*for simplicity, should be a type class*}
 
-datatype ord = LESS | EQUAL | GREATER
+datatype_new ord = LESS | EQUAL | GREATER
 
 definition "ord i j = (if i<j then LESS else if i=j then EQUAL else GREATER)"
 
-datatype 'a tree23 =
+datatype_new 'a tree23 =
   Empty |
   Branch2 "'a tree23" "key * 'a" "'a tree23" |
   Branch3 "'a tree23" "key * 'a" "'a tree23" "key * 'a" "'a tree23"
 
-datatype 'a growth =
+datatype_new 'a growth =
   Stay "'a tree23" |
   Sprout "'a tree23" "key * 'a" "'a tree23"
 
@@ -402,7 +402,7 @@
 text{* This is a little test harness and should be commented out once the
 above functions have been proved correct. *}
 
-datatype 'a act = Add int 'a | Del int
+datatype_new 'a act = Add int 'a | Del int
 
 fun exec where
 "exec [] t = t" |