src/HOL/IMP/Abs_Int_ITP/Abs_Int2_ivl_ITP.thy
changeset 58249 180f1b3508ed
parent 57512 cc97b347b301
child 58310 91ea607a34d8
--- a/src/HOL/IMP/Abs_Int_ITP/Abs_Int2_ivl_ITP.thy	Tue Sep 09 17:51:07 2014 +0200
+++ b/src/HOL/IMP/Abs_Int_ITP/Abs_Int2_ivl_ITP.thy	Tue Sep 09 20:51:36 2014 +0200
@@ -6,7 +6,7 @@
 
 subsection "Interval Analysis"
 
-datatype ivl = I "int option" "int option"
+datatype_new ivl = I "int option" "int option"
 
 definition "\<gamma>_ivl i = (case i of
   I (Some l) (Some h) \<Rightarrow> {l..h} |