--- 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 *}