src/CCL/CCL.thy
changeset 59498 50b60f501b05
parent 58977 9576b510f6a2
child 59499 14095f771781
--- a/src/CCL/CCL.thy	Tue Feb 10 14:29:36 2015 +0100
+++ b/src/CCL/CCL.thy	Tue Feb 10 14:48:26 2015 +0100
@@ -205,7 +205,7 @@
       val inj_lemmas = maps mk_inj_lemmas rews
     in
       CHANGED (REPEAT (ares_tac [@{thm iffI}, @{thm allI}, @{thm conjI}] i ORELSE
-        eresolve_tac inj_lemmas i ORELSE
+        eresolve_tac ctxt inj_lemmas i ORELSE
         asm_simp_tac (ctxt addsimps rews) i))
     end;
 *}
@@ -267,7 +267,7 @@
   let
     fun mk_raw_dstnct_thm rls s =
       Goal.prove_global @{theory} [] [] (Syntax.read_prop_global @{theory} s)
-        (fn _ => rtac @{thm notI} 1 THEN eresolve_tac rls 1)
+        (fn {context = ctxt, ...} => rtac @{thm notI} 1 THEN eresolve_tac ctxt rls 1)
   in map (mk_raw_dstnct_thm caseB_lemmas)
     (mk_dstnct_rls @{theory} ["bot","true","false","pair","lambda"]) end