src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML
changeset 41151 d58157bb1ae7
parent 41140 9c68004b8c9d
child 41152 4a7410be4dfc
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML	Wed Dec 15 11:26:29 2010 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML	Wed Dec 15 11:26:29 2010 +0100
@@ -540,15 +540,16 @@
       case outcome of
         NONE =>
         let
-          val method =
+          val (method, settings) =
             if can_apply_metis debug state subgoal (map snd used_facts) then
-              "metis"
+              ("metis", "")
             else
-              "smt"
+              ("smt", if suffix = SMT_Config.solver_of @{context} then ""
+                      else "smt_solver = " ^ maybe_quote suffix)
         in
           try_command_line (proof_banner auto)
-                           (apply_on_subgoal subgoal subgoal_count ^
-                            command_call method (map fst other_lemmas)) ^
+              (apply_on_subgoal settings subgoal subgoal_count ^
+               command_call method (map fst other_lemmas)) ^
           minimize_line minimize_command
                         (map fst (other_lemmas @ chained_lemmas))
         end