src/HOL/Bali/Conform.thy
changeset 24783 5a3e336a2e37
parent 16417 9bc16273c2d4
child 30235 58d147683393
--- a/src/HOL/Bali/Conform.thy	Sun Sep 30 16:53:08 2007 +0200
+++ b/src/HOL/Bali/Conform.thy	Sun Sep 30 21:55:15 2007 +0200
@@ -17,7 +17,7 @@
 \end{itemize}
 *}
 
-types	env_ = "prog \<times> (lname, ty) table" (* same as env of WellType.thy *)
+types	env' = "prog \<times> (lname, ty) table" (* same as env of WellType.thy *)
 
 
 section "extension of global store"
@@ -388,7 +388,7 @@
 
 constdefs
 
-  conforms :: "state \<Rightarrow> env_ \<Rightarrow> bool"          (     "_\<Colon>\<preceq>_"   [71,71]      70)
+  conforms :: "state \<Rightarrow> env' \<Rightarrow> bool"          (     "_\<Colon>\<preceq>_"   [71,71]      70)
    "xs\<Colon>\<preceq>E \<equiv> let (G, L) = E; s = snd xs; l = locals s in
     (\<forall>r. \<forall>obj\<in>globs s r:           G,s\<turnstile>obj   \<Colon>\<preceq>\<surd>r) \<and>
                 \<spacespace>                   G,s\<turnstile>l    [\<sim>\<Colon>\<preceq>]L\<spacespace> \<and>