src/HOL/IMPP/Hoare.thy
changeset 58310 91ea607a34d8
parent 58254 c1c65a805d0f
child 58889 5b7a9633cfa8
--- a/src/HOL/IMPP/Hoare.thy	Thu Sep 11 19:26:59 2014 +0200
+++ b/src/HOL/IMPP/Hoare.thy	Thu Sep 11 19:32:36 2014 +0200
@@ -28,7 +28,7 @@
   peek_and :: "'a assn => (state => bool) => 'a assn" (infixr "&>" 35) where
   "peek_and P p = (%Z s. P Z s & p s)"
 
-datatype_new 'a triple =
+datatype 'a triple =
   triple "'a assn"  com  "'a assn"       ("{(1_)}./ (_)/ .{(1_)}" [3,60,3] 58)
 
 definition