src/HOL/Tools/Sledgehammer/sledgehammer_prover_tactic.ML
changeset 82620 2d854f1cd830
parent 82576 a310d5b6c696
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_prover_tactic.ML	Sun May 11 12:05:10 2025 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_prover_tactic.ML	Mon May 12 13:02:52 2025 +0200
@@ -98,9 +98,17 @@
         NONE => (found_something name; map fst facts)
       | SOME _ => [])
 
-    val message = fn _ =>
+    val message = fn preplay_outcome =>
       (case outcome of
-        NONE => try_command_line (proof_banner mode name) (Played run_time) command
+        NONE =>
+        let
+          val banner = proof_banner mode name
+        in
+          (case preplay_outcome of
+            NONE => try_command_line banner (Played run_time) command
+          | SOME preplay_result =>
+              one_line_proof_text (preplay_result, banner, subgoal, subgoal_count))
+        end
       | SOME failure => string_of_atp_failure failure)
   in
     {outcome = outcome, used_facts = used_facts, used_from = facts,