src/HOL/Bali/AxSound.thy
changeset 12937 0c4fd7529467
parent 12925 99131847fb93
child 13337 f75dfc606ac7
--- a/src/HOL/Bali/AxSound.thy	Mon Feb 25 20:46:09 2002 +0100
+++ b/src/HOL/Bali/AxSound.thy	Mon Feb 25 20:48:14 2002 +0100
@@ -247,11 +247,11 @@
 done
 
 corollary evaln_type_sound:
-      (assumes evaln: "G\<turnstile>s0 \<midarrow>t\<succ>\<midarrow>n\<rightarrow> (v,s1)" and
-                  wt: "\<lparr>prg=G,cls=accC,lcl=L\<rparr>\<turnstile>t\<Colon>T" and
-             conf_s0: "s0\<Colon>\<preceq>(G,L)" and
-                  wf: "wf_prog G"                         
-      ) "s1\<Colon>\<preceq>(G,L) \<and>  (normal s1 \<longrightarrow> G,L,store s1\<turnstile>t\<succ>v\<Colon>\<preceq>T) \<and> 
+  assumes evaln: "G\<turnstile>s0 \<midarrow>t\<succ>\<midarrow>n\<rightarrow> (v,s1)" and
+             wt: "\<lparr>prg=G,cls=accC,lcl=L\<rparr>\<turnstile>t\<Colon>T" and
+        conf_s0: "s0\<Colon>\<preceq>(G,L)" and
+             wf: "wf_prog G"                         
+  shows "s1\<Colon>\<preceq>(G,L) \<and>  (normal s1 \<longrightarrow> G,L,store s1\<turnstile>t\<succ>v\<Colon>\<preceq>T) \<and> 
          (error_free s0 = error_free s1)"
 proof -
   from evaln wt conf_s0 wf