src/HOL/SPARK/Manual/Complex_Types.thy
changeset 58310 91ea607a34d8
parent 58130 5e9170812356
child 63167 0909deb8059b
--- a/src/HOL/SPARK/Manual/Complex_Types.thy	Thu Sep 11 19:26:59 2014 +0200
+++ b/src/HOL/SPARK/Manual/Complex_Types.thy	Thu Sep 11 19:32:36 2014 +0200
@@ -2,7 +2,7 @@
 imports "../SPARK"
 begin
 
-datatype_new day = Mon | Tue | Wed | Thu | Fri | Sat | Sun
+datatype day = Mon | Tue | Wed | Thu | Fri | Sat | Sun
 
 record two_fields =
   Field1 :: "int \<times> day \<Rightarrow> int"