src/HOL/Bali/TypeSafe.thy
changeset 19796 d86e7b1fc472
parent 18585 5d379fe2eb74
child 21765 89275a3ed7be
--- a/src/HOL/Bali/TypeSafe.thy	Tue Jun 06 19:24:05 2006 +0200
+++ b/src/HOL/Bali/TypeSafe.thy	Tue Jun 06 20:42:25 2006 +0200
@@ -3878,7 +3878,7 @@
                                P L accC s1 \<langle>c2\<rangle>\<^sub>s \<diamondsuit> s2\<rbrakk> \<Longrightarrow> Q
                         \<rbrakk> \<Longrightarrow> Q 
                   \<rbrakk>\<Longrightarrow> P L accC (Norm s0) \<langle>c1;; c2\<rangle>\<^sub>s \<diamondsuit> s2" 
-    and    if: "\<And> b c1 c2 e s0 s1 s2 L accC E.
+    and  "if": "\<And> b c1 c2 e s0 s1 s2 L accC E.
                 \<lbrakk>G\<turnstile>Norm s0 \<midarrow>e-\<succ>b\<rightarrow> s1;
                  G\<turnstile>s1 \<midarrow>(if the_Bool b then c1 else c2)\<rightarrow> s2;
                  \<lparr>prg=G,cls=accC,lcl=L\<rparr>\<turnstile>e\<Colon>-PrimT Boolean;
@@ -4030,7 +4030,7 @@
     }
     with eval_e eval_then_else wt_e wt_then_else da_e P_e
     show ?case
-      by (rule if) iprover+
+      by (rule "if") iprover+
   next
     oops