src/HOL/Quickcheck_Exhaustive.thy
changeset 58310 91ea607a34d8
parent 58152 6fe60a9a5bad
child 58334 7553a1bcecb7
--- a/src/HOL/Quickcheck_Exhaustive.thy	Thu Sep 11 19:26:59 2014 +0200
+++ b/src/HOL/Quickcheck_Exhaustive.thy	Thu Sep 11 19:32:36 2014 +0200
@@ -574,8 +574,8 @@
 where
   "pos_bound_cps_if b = (if b then pos_bound_cps_single () else pos_bound_cps_empty)"
 
-datatype_new (dead 'a) unknown = Unknown | Known 'a
-datatype_new (dead 'a) three_valued = Unknown_value | Value 'a | No_value
+datatype (dead 'a) unknown = Unknown | Known 'a
+datatype (dead 'a) three_valued = Unknown_value | Value 'a | No_value
 
 type_synonym 'a neg_bound_cps = "('a unknown => term list three_valued) => natural => term list three_valued"