tuned;
authorwenzelm
Mon, 10 Jun 2024 14:04:52 +0200
changeset 80327 e4e643705d90
parent 80326 53f12ab896e6
child 80328 559909bd7715
tuned;
src/HOL/Tools/Sledgehammer/sledgehammer_isar_preplay.ML
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_isar_preplay.ML	Mon Jun 10 12:44:49 2024 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_isar_preplay.ML	Mon Jun 10 14:04:52 2024 +0200
@@ -94,7 +94,7 @@
     val assms = Pretty.enum " and " "using " " shows " (map (Thm.pretty_thm ctxt) assms)
     val concl = Syntax.pretty_term ctxt concl
   in
-    tracing (Pretty.string_of (Pretty.blk (2, Pretty.breaks [time, assms, concl])))
+    tracing (Pretty.string_of (Pretty.block (Pretty.breaks [time, assms, concl])))
   end
 
 fun take_time timeout tac arg =