src/HOL/Bali/Eval.thy
changeset 59498 50b60f501b05
parent 58887 38db8ddc0f57
child 61989 ba8c284d4725
--- a/src/HOL/Bali/Eval.thy	Tue Feb 10 14:29:36 2015 +0100
+++ b/src/HOL/Bali/Eval.thy	Tue Feb 10 14:48:26 2015 +0100
@@ -1163,7 +1163,7 @@
   "G\<turnstile>s \<midarrow>t\<succ>\<rightarrow> (w, s') \<Longrightarrow> (\<forall>w' s''. G\<turnstile>s \<midarrow>t\<succ>\<rightarrow> (w', s'') \<longrightarrow> w' = w \<and> s'' = s')"
 apply (erule eval_induct)
 apply (tactic {* ALLGOALS (EVERY'
-      [strip_tac, rotate_tac ~1, eresolve_tac @{thms eval_elim_cases}]) *})
+      [strip_tac @{context}, rotate_tac ~1, eresolve_tac @{context} @{thms eval_elim_cases}]) *})
 (* 31 subgoals *)
 prefer 28 (* Try *) 
 apply (simp (no_asm_use) only: split add: split_if_asm)