src/HOL/Bali/AxCompl.thy
changeset 26932 c398a3866082
parent 24783 5a3e336a2e37
child 31945 d5f186aa0bed
--- a/src/HOL/Bali/AxCompl.thy	Sat May 17 15:31:42 2008 +0200
+++ b/src/HOL/Bali/AxCompl.thy	Sat May 17 21:46:22 2008 +0200
@@ -970,7 +970,7 @@
   fix l show "abrupt s2 \<noteq> Some (Jump (Break l)) \<and>  
               abrupt s2 \<noteq> Some (Jump (Cont l))"
   proof -
-    from clsD have wt_init: "\<lparr>prg=G, cls=accC, lcl=L\<rparr>\<turnstile>(Init D)\<Colon>\<surd>"
+    fix accC from clsD have wt_init: "\<lparr>prg=G, cls=accC, lcl=L\<rparr>\<turnstile>(Init D)\<Colon>\<surd>"
       by auto
     from eval_init wf
     have s1_no_jmp: "\<And> j. abrupt s1 \<noteq> Some (Jump j)"