src/HOL/MicroJava/J/Decl.thy
changeset 35416 d8d7d1b785af
parent 18551 be0705186ff5
child 35431 8758fe1fc9f8
--- a/src/HOL/MicroJava/J/Decl.thy	Wed Feb 24 11:55:52 2010 +0100
+++ b/src/HOL/MicroJava/J/Decl.thy	Mon Mar 01 13:40:23 2010 +0100
@@ -1,5 +1,4 @@
 (*  Title:      HOL/MicroJava/J/Decl.thy
-    ID:         $Id$
     Author:     David von Oheimb
     Copyright   1999 Technische Universitaet Muenchen
 *)
@@ -32,11 +31,10 @@
   "prog  c" <= (type) "(c cdecl) list"
 
 
-constdefs
-  "class" :: "'c prog => (cname \<rightharpoonup> 'c class)"
+definition "class" :: "'c prog => (cname \<rightharpoonup> 'c class)" where
   "class \<equiv> map_of"
 
-  is_class :: "'c prog => cname => bool"
+definition is_class :: "'c prog => cname => bool" where
   "is_class G C \<equiv> class G C \<noteq> None"
 
 
@@ -46,10 +44,8 @@
 apply (rule finite_dom_map_of)
 done
 
-consts
-  is_type :: "'c prog => ty    => bool"
-primrec
+primrec is_type :: "'c prog => ty => bool" where
   "is_type G (PrimT pt) = True"
-  "is_type G (RefT t) = (case t of NullT => True | ClassT C => is_class G C)"
+| "is_type G (RefT t) = (case t of NullT => True | ClassT C => is_class G C)"
 
 end