src/Provers/Arith/fast_lin_arith.ML
changeset 35230 be006fbcfb96
parent 33519 e31a85f92ce9
child 35693 d58a4ac1ca1c
--- a/src/Provers/Arith/fast_lin_arith.ML	Fri Feb 19 09:35:18 2010 +0100
+++ b/src/Provers/Arith/fast_lin_arith.ML	Fri Feb 19 11:49:44 2010 +0100
@@ -56,7 +56,7 @@
   val pre_decomp: Proof.context -> typ list * term list -> (typ list * term list) list
 
   (*preprocessing, performed on the goal -- must do the same as 'pre_decomp':*)
-  val pre_tac: Proof.context -> int -> tactic
+  val pre_tac: simpset -> int -> tactic
 
   (*the limit on the number of ~= allowed; because each ~= is split
     into two cases, this can lead to an explosion*)
@@ -792,7 +792,7 @@
       (* rewrite "[| A1; ...; An |] ==> B" to "[| A1; ...; An; ~B |] ==> False" *)
       DETERM (resolve_tac [LA_Logic.notI, LA_Logic.ccontr] i) THEN
       (* user-defined preprocessing of the subgoal *)
-      DETERM (LA_Data.pre_tac ctxt i) THEN
+      DETERM (LA_Data.pre_tac ss i) THEN
       PRIMITIVE (trace_thm ctxt "State after pre_tac:") THEN
       (* prove every resulting subgoal, using its justification *)
       EVERY (map just1 justs)