src/HOL/Presburger.thy
changeset 24094 6db35c14146d
parent 24075 366d4d234814
child 24404 317b207bc1ab
--- a/src/HOL/Presburger.thy	Tue Jul 31 19:40:24 2007 +0200
+++ b/src/HOL/Presburger.thy	Tue Jul 31 19:40:25 2007 +0200
@@ -441,10 +441,9 @@
 
 declaration {* fn _ =>
   arith_tactic_add
-    (mk_arith_tactic "presburger" (fn i => fn st =>
+    (mk_arith_tactic "presburger" (fn ctxt => fn i => fn st =>
        (warning "Trying Presburger arithmetic ...";   
-    Presburger.cooper_tac true [] [] ((ProofContext.init o theory_of_thm) st) i st)))
-  (* FIXME!!!!!!! get the right context!!*)	
+    Presburger.cooper_tac true [] [] ctxt i st)))
 *}
 
 method_setup presburger = {*