src/LCF/LCF.thy
changeset 59498 50b60f501b05
parent 58977 9576b510f6a2
child 59755 f8d164ab0dc1
--- a/src/LCF/LCF.thy	Tue Feb 10 14:29:36 2015 +0100
+++ b/src/LCF/LCF.thy	Tue Feb 10 14:48:26 2015 +0100
@@ -322,7 +322,7 @@
   Scan.lift Args.name_inner_syntax >> (fn v => fn ctxt =>
     SIMPLE_METHOD' (fn i =>
       res_inst_tac ctxt [(("f", 0), v)] @{thm induct} i THEN
-      REPEAT (resolve_tac @{thms adm_lemmas} i)))
+      REPEAT (resolve_tac ctxt @{thms adm_lemmas} i)))
 *}
 
 lemma least_FIX: "f(p) = p \<Longrightarrow> FIX(f) << p"
@@ -381,7 +381,7 @@
 ML {*
 fun induct2_tac ctxt (f, g) i =
   res_inst_tac ctxt [(("f", 0), f), (("g", 0), g)] @{thm induct2} i THEN
-  REPEAT(resolve_tac @{thms adm_lemmas} i)
+  REPEAT(resolve_tac ctxt @{thms adm_lemmas} i)
 *}
 
 end