src/HOL/IMP/Abs_Int_ITP/Abs_Int1_parity_ITP.thy
changeset 58249 180f1b3508ed
parent 55600 3c7610b8dcfc
child 58310 91ea607a34d8
--- a/src/HOL/IMP/Abs_Int_ITP/Abs_Int1_parity_ITP.thy	Tue Sep 09 17:51:07 2014 +0200
+++ b/src/HOL/IMP/Abs_Int_ITP/Abs_Int1_parity_ITP.thy	Tue Sep 09 20:51:36 2014 +0200
@@ -6,7 +6,7 @@
 
 subsection "Parity Analysis"
 
-datatype parity = Even | Odd | Either
+datatype_new parity = Even | Odd | Either
 
 text{* Instantiation of class @{class preord} with type @{typ parity}: *}