src/HOL/Tools/Sledgehammer/sledgehammer_prover_atp.ML
changeset 59172 d1c500e0a722
parent 58843 521cea5fa777
child 59577 012c6165bbd2
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_prover_atp.ML	Sun Dec 21 22:49:40 2014 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_prover_atp.ML	Mon Dec 22 14:33:53 2014 +0100
@@ -351,10 +351,9 @@
       with_cleanup clean_up run () |> tap export
 
     val important_message =
-      if mode = Normal andalso random_range 0 (atp_important_message_keep_quotient - 1) = 0 then
-        extract_important_message output
-      else
-        ""
+      if mode = Normal andalso Random.random_range 0 (atp_important_message_keep_quotient - 1) = 0
+      then extract_important_message output
+      else ""
 
     val (used_facts, preferred_methss, message) =
       (case outcome of