src/HOL/Old_Number_Theory/IntPrimes.thy
changeset 59498 50b60f501b05
parent 58889 5b7a9633cfa8
child 61382 efac889fccbc
--- a/src/HOL/Old_Number_Theory/IntPrimes.thy	Tue Feb 10 14:29:36 2015 +0100
+++ b/src/HOL/Old_Number_Theory/IntPrimes.thy	Tue Feb 10 14:48:26 2015 +0100
@@ -399,7 +399,7 @@
     zgcd a n = 1 ==> \<exists>!x. 0 \<le> x \<and> x < n \<and> [a * x = b] (mod n)"
   apply auto
    apply (rule_tac [2] zcong_zless_imp_eq)
-       apply (tactic {* stac (@{thm zcong_cancel2} RS sym) 6 *})
+       apply (tactic {* stac @{context} (@{thm zcong_cancel2} RS sym) 6 *})
          apply (rule_tac [8] zcong_trans)
           apply (simp_all (no_asm_simp))
    prefer 2