src/HOL/HOLCF/Discrete.thy
changeset 58249 180f1b3508ed
parent 42151 4da4fc77664b
child 58310 91ea607a34d8
--- a/src/HOL/HOLCF/Discrete.thy	Tue Sep 09 17:51:07 2014 +0200
+++ b/src/HOL/HOLCF/Discrete.thy	Tue Sep 09 20:51:36 2014 +0200
@@ -8,7 +8,7 @@
 imports Cont
 begin
 
-datatype 'a discr = Discr "'a :: type"
+datatype_new 'a discr = Discr "'a :: type"
 
 subsection {* Discrete cpo class instance *}