src/HOL/MicroJava/J/Type.thy
changeset 58310 91ea607a34d8
parent 58249 180f1b3508ed
child 58886 8a6cac7c7247
--- a/src/HOL/MicroJava/J/Type.thy	Thu Sep 11 19:26:59 2014 +0200
+++ b/src/HOL/MicroJava/J/Type.thy	Thu Sep 11 19:32:36 2014 +0200
@@ -45,14 +45,14 @@
 end
 
  -- "exceptions"
-datatype_new 
+datatype 
   xcpt   
   = NullPointer
   | ClassCast
   | OutOfMemory
 
 -- "class names"
-datatype_new cname  
+datatype cname  
   = Object 
   | Xcpt xcpt 
   | Cname cnam 
@@ -128,23 +128,23 @@
 end
 
 -- "names for @{text This} pointer and local/field variables"
-datatype_new vname 
+datatype vname 
   = This
   | VName vnam
 
 -- "primitive type, cf. 4.2"
-datatype_new prim_ty 
+datatype prim_ty 
   = Void          -- "'result type' of void methods"
   | Boolean
   | Integer
 
 -- "reference type, cf. 4.3"
-datatype_new ref_ty   
+datatype ref_ty   
   = NullT         -- "null type, cf. 4.1"
   | ClassT cname  -- "class type"
 
 -- "any type, cf. 4.1"
-datatype_new ty 
+datatype ty 
   = PrimT prim_ty -- "primitive type"
   | RefT  ref_ty  -- "reference type"