src/HOL/IMP/Abs_Int_Den/Abs_Int_den1_ivl.thy
changeset 58310 91ea607a34d8
parent 58249 180f1b3508ed
child 58410 6d46ad54a2ab
--- a/src/HOL/IMP/Abs_Int_Den/Abs_Int_den1_ivl.thy	Thu Sep 11 19:26:59 2014 +0200
+++ b/src/HOL/IMP/Abs_Int_Den/Abs_Int_den1_ivl.thy	Thu Sep 11 19:32:36 2014 +0200
@@ -6,7 +6,7 @@
 
 subsection "Interval Analysis"
 
-datatype_new ivl = I "int option" "int option"
+datatype ivl = I "int option" "int option"
 
 text{* We assume an important invariant: arithmetic operations are never
 applied to empty intervals @{term"I (Some i) (Some j)"} with @{term"j <