src/Pure/Pure.thy
changeset 76077 0f48e873e187
parent 75687 c8dc5d1adc7b
child 76923 8a66a88cd5dc
--- a/src/Pure/Pure.thy	Wed Sep 07 11:17:46 2022 +0200
+++ b/src/Pure/Pure.thy	Wed Sep 07 11:25:49 2022 +0200
@@ -1302,7 +1302,7 @@
   Outer_Syntax.command \<^command_keyword>\<open>print_state\<close>
     "print current proof state (if present)"
     (opt_modes >> (fn modes =>
-      Toplevel.keep (Print_Mode.with_modes modes (Output.state o Toplevel.string_of_state))));
+      Toplevel.keep (Print_Mode.with_modes modes (Output.writeln o Toplevel.string_of_state))));
 
 val _ =
   Outer_Syntax.command \<^command_keyword>\<open>welcome\<close> "print welcome message"