src/HOL/Lattice/Orders.thy
changeset 58310 91ea607a34d8
parent 58249 180f1b3508ed
child 58879 143c85e3cdb5
--- a/src/HOL/Lattice/Orders.thy	Thu Sep 11 19:26:59 2014 +0200
+++ b/src/HOL/Lattice/Orders.thy	Thu Sep 11 19:32:36 2014 +0200
@@ -46,7 +46,7 @@
   of the original one.
 *}
 
-datatype_new 'a dual = dual 'a
+datatype 'a dual = dual 'a
 
 primrec undual :: "'a dual \<Rightarrow> 'a" where
   undual_dual: "undual (dual x) = x"