src/HOL/MicroJava/J/Conform.thy
changeset 24783 5a3e336a2e37
parent 16417 9bc16273c2d4
child 26342 0f65fa163304
--- a/src/HOL/MicroJava/J/Conform.thy	Sun Sep 30 16:53:08 2007 +0200
+++ b/src/HOL/MicroJava/J/Conform.thy	Sun Sep 30 21:55:15 2007 +0200
@@ -8,7 +8,7 @@
 
 theory Conform imports State WellType Exceptions begin
 
-types 'c env_ = "'c prog \<times> (vname \<rightharpoonup> ty)"  -- "same as @{text env} of @{text WellType.thy}"
+types 'c env' = "'c prog \<times> (vname \<rightharpoonup> ty)"  -- "same as @{text env} of @{text WellType.thy}"
 
 constdefs
 
@@ -32,7 +32,7 @@
   xconf :: "aheap \<Rightarrow> val option \<Rightarrow> bool"
   "xconf hp vo  == preallocated hp \<and> (\<forall> v. (vo = Some v) \<longrightarrow> (\<exists> xc. v = (Addr (XcptRef xc))))"
 
-  conforms :: "xstate => java_mb env_ => bool" ("_ ::<= _" [51,51] 50)
+  conforms :: "xstate => java_mb env' => bool" ("_ ::<= _" [51,51] 50)
  "s::<=E == prg E|-h heap (store s) [ok] \<and> 
             prg E,heap (store s)|-locals (store s)[::<=]localT E \<and> 
             xconf (heap (store s)) (abrupt s)"
@@ -54,7 +54,7 @@
   hconf    :: "'c prog => aheap => bool"
               ("_ \<turnstile>h _ \<surd>" [51,51] 50)
 
-  conforms :: "state => java_mb env_ => bool"
+  conforms :: "state => java_mb env' => bool"
               ("_ ::\<preceq> _" [51,51] 50)