src/HOL/Divides.thy
changeset 28262 aa7ca36d67fd
parent 27676 55676111ed69
child 28562 4e74209f113e
--- a/src/HOL/Divides.thy	Wed Sep 17 21:27:03 2008 +0200
+++ b/src/HOL/Divides.thy	Wed Sep 17 21:27:08 2008 +0200
@@ -371,7 +371,7 @@
 
 structure CancelDivMod = CancelDivModFun(CancelDivModData);
 
-val cancel_div_mod_proc = Simplifier.simproc @{theory}
+val cancel_div_mod_proc = Simplifier.simproc (the_context ())
   "cancel_div_mod" ["(m::nat) + n"] (K CancelDivMod.proc);
 
 Addsimprocs[cancel_div_mod_proc];