src/Tools/solve_direct.ML
changeset 58892 20aa19ecf2cc
parent 58843 521cea5fa777
child 58893 9e0ecb66d6a7
--- a/src/Tools/solve_direct.ML	Mon Nov 03 09:25:23 2014 +0100
+++ b/src/Tools/solve_direct.ML	Mon Nov 03 14:31:15 2014 +0100
@@ -15,7 +15,7 @@
   val noneN: string
   val unknownN: string
   val max_solutions: int Unsynchronized.ref
-  val solve_direct: Proof.state -> bool * (string * Proof.state)
+  val solve_direct: Proof.state -> bool * (string * string list)
 end;
 
 structure Solve_Direct: SOLVE_DIRECT =
@@ -76,22 +76,17 @@
     (case try seek_against_goal () of
       SOME (SOME results) =>
         (someN,
-          state |>
-            (if mode = Auto_Try then
-               Proof.goal_message
-                 (fn () =>
-                   Pretty.markup Markup.information (message results))
-             else
-               tap (fn _ =>
-                 writeln (Pretty.string_of (Pretty.chunks (message results))))))
+          if mode = Auto_Try then
+            [Pretty.string_of (Pretty.markup Markup.information (message results))]
+          else (writeln (Pretty.string_of (Pretty.chunks (message results))); []))
     | SOME NONE =>
         (if mode = Normal then writeln "No proof found."
          else ();
-         (noneN, state))
+         (noneN, []))
     | NONE =>
         (if mode = Normal then writeln "An error occurred."
          else ();
-         (unknownN, state)))
+         (unknownN, [])))
   end
   |> `(fn (outcome_code, _) => outcome_code = someN);