src/HOL/Divides.thy
changeset 51717 9e7d1c139569
parent 51299 30b014246e21
child 52398 656e5e171f19
--- a/src/HOL/Divides.thy	Tue Apr 16 17:54:14 2013 +0200
+++ b/src/HOL/Divides.thy	Thu Apr 18 17:07:01 2013 +0200
@@ -1643,12 +1643,12 @@
   val simps = @{thms arith_simps} @ @{thms rel_simps} @
     map (fn th => th RS sym) [@{thm numeral_1_eq_1}]
   fun prove ctxt goal = Goal.prove ctxt [] [] (HOLogic.mk_Trueprop goal)
-    (K (ALLGOALS (full_simp_tac (HOL_basic_ss addsimps simps))));
-  fun binary_proc proc ss ct =
+    (K (ALLGOALS (full_simp_tac (put_simpset HOL_basic_ss ctxt addsimps simps))));
+  fun binary_proc proc ctxt ct =
     (case Thm.term_of ct of
       _ $ t $ u =>
       (case try (pairself (`(snd o HOLogic.dest_number))) (t, u) of
-        SOME args => proc (Simplifier.the_context ss) args
+        SOME args => proc ctxt args
       | NONE => NONE)
     | _ => NONE);
 in