src/HOL/Tools/Sledgehammer/sledgehammer_filter.ML
changeset 41491 a2ad5b824051
parent 41336 0ea5b9c7d233
child 41767 44b2a0385001
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_filter.ML	Mon Jan 10 15:30:17 2011 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_filter.ML	Mon Jan 10 15:45:46 2011 +0100
@@ -95,7 +95,7 @@
 
 fun make_name reserved multi j name =
   (name |> needs_quoting reserved name ? quote) ^
-  (if multi then "(" ^ Int.toString j ^ ")" else "")
+  (if multi then "(" ^ string_of_int j ^ ")" else "")
 
 fun explode_interval _ (Facts.FromTo (i, j)) = i upto j
   | explode_interval max (Facts.From i) = i upto i + max - 1
@@ -482,8 +482,8 @@
       chop max_imperfect imperfect |>> append perfect |>> chop remaining_max
   in
     trace_msg (fn () =>
-        "Actually passed (" ^ Int.toString (length accepts) ^ " of " ^
-        Int.toString (length candidates) ^ "): " ^
+        "Actually passed (" ^ string_of_int (length accepts) ^ " of " ^
+        string_of_int (length candidates) ^ "): " ^
         (accepts |> map (fn ((((name, _), _), _), weight) =>
                             name () ^ " [" ^ Real.toString weight ^ "]")
                  |> commas));
@@ -612,7 +612,7 @@
                  accepts |> needs_ext is_built_in_const accepts
                             ? add_facts @{thms ext})
           |> tap (fn accepts => trace_msg (fn () =>
-                      "Total relevant: " ^ Int.toString (length accepts)))
+                      "Total relevant: " ^ string_of_int (length accepts)))
   end
 
 
@@ -886,7 +886,7 @@
       |> rearrange_facts ctxt (respect_no_atp andalso not only)
       |> uniquify
   in
-    trace_msg (fn () => "Considering " ^ Int.toString (length facts) ^
+    trace_msg (fn () => "Considering " ^ string_of_int (length facts) ^
                         " facts");
     (if only orelse threshold1 < 0.0 then
        facts