src/HOL/Decision_Procs/Approximation.thy
changeset 59498 50b60f501b05
parent 59058 a78612c67ec0
child 59580 cbc38731d42f
--- a/src/HOL/Decision_Procs/Approximation.thy	Tue Feb 10 14:29:36 2015 +0100
+++ b/src/HOL/Decision_Procs/Approximation.thy	Tue Feb 10 14:48:26 2015 +0100
@@ -3699,7 +3699,7 @@
                       etac @{thm meta_eqE},
                       rtac @{thm impI}] i)
       THEN Subgoal.FOCUS (fn {prems, ...} => reorder_bounds_tac prems i) ctxt i
-      THEN DETERM (TRY (filter_prems_tac (K false) i))
+      THEN DETERM (TRY (filter_prems_tac ctxt (K false) i))
       THEN DETERM (Reification.tac ctxt form_equations NONE i)
       THEN rewrite_interpret_form_tac ctxt prec splitting taylor i
       THEN gen_eval_tac (approximation_conv ctxt) ctxt i))