src/Tools/quickcheck.ML
changeset 43029 3e060b1c844b
parent 43024 58150aa44941
child 43112 3117573292b8
--- a/src/Tools/quickcheck.ML	Fri May 27 10:30:08 2011 +0200
+++ b/src/Tools/quickcheck.ML	Fri May 27 10:30:08 2011 +0200
@@ -638,22 +638,22 @@
     | SOME results =>
         let
           val msg = pretty_counterex_and_reports ctxt auto results
-                    |> not auto ? tap (Output.urgent_message o Pretty.string_of)
         in
           if exists found_counterexample results then
             (genuineN,
-             state |> (if auto then
-                         Proof.goal_message (K (Pretty.chunks [Pretty.str "",
-                             Pretty.mark Markup.hilite msg]))
-                       else
-                         I))
+             state
+             |> (if auto then
+                   Proof.goal_message (K (Pretty.chunks [Pretty.str "",
+                       Pretty.mark Markup.hilite msg]))
+                 else
+                   tap (fn _ => Output.urgent_message (Pretty.string_of msg))))
           else
             (noneN, state)
         end
   end
   |> `(fn (outcome_code, _) => outcome_code = genuineN)
 
-val setup = Try.register_tool (quickcheckN, (30, auto, try_quickcheck))
+val setup = Try.register_tool (quickcheckN, (20, auto, try_quickcheck))
 
 end;