src/HOL/MicroJava/J/Term.thy
changeset 58310 91ea607a34d8
parent 58263 6c907aad90ba
child 58886 8a6cac7c7247
--- a/src/HOL/MicroJava/J/Term.thy	Thu Sep 11 19:26:59 2014 +0200
+++ b/src/HOL/MicroJava/J/Term.thy	Thu Sep 11 19:32:36 2014 +0200
@@ -6,9 +6,9 @@
 
 theory Term imports Value begin
 
-datatype_new binop = Eq | Add    -- "function codes for binary operation"
+datatype binop = Eq | Add    -- "function codes for binary operation"
 
-datatype_new expr
+datatype expr
   = NewC cname               -- "class instance creation"
   | Cast cname expr          -- "type cast"
   | Lit val                  -- "literal value, also references"
@@ -23,7 +23,7 @@
 
 datatype_compat expr
 
-datatype_new stmt
+datatype stmt
   = Skip                     -- "empty statement"
   | Expr expr                -- "expression statement"
   | Comp stmt stmt       ("_;; _"             [61,60]60)