src/HOL/Hoare/Heap.thy
changeset 58310 91ea607a34d8
parent 58249 180f1b3508ed
child 62042 6c6ccf573479
--- a/src/HOL/Hoare/Heap.thy	Thu Sep 11 19:26:59 2014 +0200
+++ b/src/HOL/Hoare/Heap.thy	Thu Sep 11 19:32:36 2014 +0200
@@ -10,7 +10,7 @@
 
 subsection "References"
 
-datatype_new 'a ref = Null | Ref 'a
+datatype 'a ref = Null | Ref 'a
 
 lemma not_Null_eq [iff]: "(x ~= Null) = (EX y. x = Ref y)"
   by (induct x) auto