src/Sequents/modal.ML
changeset 54742 7a86358a3c0b
parent 41449 7339f0e7c513
child 59164 ff40c53d1af9
--- a/src/Sequents/modal.ML	Fri Dec 13 23:53:02 2013 +0100
+++ b/src/Sequents/modal.ML	Sat Dec 14 17:28:05 2013 +0100
@@ -19,7 +19,7 @@
     val rule_tac   : thm list -> int ->tactic
     val step_tac   : int -> tactic
     val solven_tac : int -> int -> tactic
-    val solve_tac  : int -> tactic
+    val solve_tac  : Proof.context -> int -> tactic
 end;
 
 functor Modal_ProverFun (Modal_Rule: MODAL_PROVER_RULE) : MODAL_PROVER = 
@@ -78,7 +78,7 @@
                  ((fres_unsafe_tac n  THEN UPTOGOAL n (solven_tac d)) APPEND
                    (fres_bound_tac n  THEN UPTOGOAL n (solven_tac (d-1)))));
 
-fun solve_tac d = rewrite_goals_tac Modal_Rule.rewrite_rls THEN solven_tac d 1;
+fun solve_tac ctxt d = rewrite_goals_tac ctxt Modal_Rule.rewrite_rls THEN solven_tac d 1;
 
 fun step_tac n = 
     COND (has_fewer_prems 1) all_tac