src/HOL/MicroJava/J/Exceptions.thy
changeset 35102 cc7a0b9f938c
parent 30235 58d147683393
child 35416 d8d7d1b785af
--- a/src/HOL/MicroJava/J/Exceptions.thy	Wed Feb 10 23:53:46 2010 +0100
+++ b/src/HOL/MicroJava/J/Exceptions.thy	Thu Feb 11 00:45:02 2010 +0100
@@ -1,5 +1,4 @@
 (*  Title:      HOL/MicroJava/J/Exceptions.thy
-    ID:         $Id$
     Author:     Gerwin Klein, Martin Strecker
     Copyright   2002 Technische Universitaet Muenchen
 *)
@@ -17,11 +16,9 @@
                         (XcptRef OutOfMemory \<mapsto> blank G (Xcpt OutOfMemory))"
 
 
-consts
+abbreviation
   cname_of :: "aheap \<Rightarrow> val \<Rightarrow> cname"
-
-translations
-  "cname_of hp v" == "fst (CONST the (hp (the_Addr v)))"
+  where "cname_of hp v == fst (the (hp (the_Addr v)))"
 
 
 constdefs