src/Tools/quickcheck.ML
changeset 58843 521cea5fa777
parent 58842 22b87ab47d3b
child 58892 20aa19ecf2cc
--- a/src/Tools/quickcheck.ML	Fri Oct 31 11:18:17 2014 +0100
+++ b/src/Tools/quickcheck.ML	Fri Oct 31 11:36:41 2014 +0100
@@ -294,11 +294,11 @@
         if is_interactive then exc () else raise TimeLimit.TimeOut
   else f ();
 
-fun message ctxt s = if Config.get ctxt quiet then () else Output.urgent_message s;
+fun message ctxt s = if Config.get ctxt quiet then () else writeln s;
 
 fun verbose_message ctxt s =
   if not (Config.get ctxt quiet) andalso Config.get ctxt verbose
-  then Output.urgent_message s else ();
+  then writeln s else ();
 
 fun test_terms ctxt (limit_time, is_interactive) insts goals =
   (case active_testers ctxt of
@@ -517,7 +517,7 @@
   gen_quickcheck args i (Toplevel.proof_of state)
   |> apfst (Option.map (the o get_first response_of))
   |> (fn (r, state) =>
-      Output.urgent_message (Pretty.string_of
+      writeln (Pretty.string_of
         (pretty_counterex (Proof.context_of state) false r)));
 
 val parse_arg =
@@ -563,7 +563,7 @@
              |> (if auto then
                    Proof.goal_message (K (Pretty.mark Markup.information msg))
                  else
-                   tap (fn _ => Output.urgent_message (Pretty.string_of msg))))
+                   tap (fn _ => writeln (Pretty.string_of msg))))
           else
             (noneN, state)
         end)