src/HOL/Tools/Sledgehammer/sledgehammer_atp_translate.ML
changeset 41491 a2ad5b824051
parent 41406 062490d081b9
child 41726 1ef01508bb9b
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_atp_translate.ML	Mon Jan 10 15:30:17 2011 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_atp_translate.ML	Mon Jan 10 15:45:46 2011 +0100
@@ -143,7 +143,7 @@
 
 val presimplify_term = prop_of o Meson.presimplify oo Skip_Proof.make_thm
 
-fun concealed_bound_name j = sledgehammer_weak_prefix ^ Int.toString j
+fun concealed_bound_name j = sledgehammer_weak_prefix ^ string_of_int j
 fun conceal_bounds Ts t =
   subst_bounds (map (Free o apfst concealed_bound_name)
                     (0 upto length Ts - 1 ~~ Ts), t)
@@ -247,7 +247,7 @@
   | formula => SOME formula
 fun make_conjecture ctxt ts =
   let val last = length ts - 1 in
-    map2 (fn j => make_formula ctxt true true (Int.toString j)
+    map2 (fn j => make_formula ctxt true true (string_of_int j)
                                (if j = last then Conjecture else Hypothesis))
          (0 upto last) ts
   end