src/HOL/Tools/Sledgehammer/sledgehammer_fol_clause.ML
changeset 36063 cdc6855a6387
parent 36062 194cb6e3c13f
child 36167 c1a35be8e476
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_fol_clause.ML	Mon Mar 29 15:50:18 2010 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_fol_clause.ML	Mon Mar 29 18:44:24 2010 +0200
@@ -80,6 +80,8 @@
 structure Sledgehammer_FOL_Clause : SLEDGEHAMMER_FOL_CLAUSE =
 struct
 
+open Sledgehammer_Util
+
 val schematic_var_prefix = "V_";
 val fixed_var_prefix = "v_";
 
@@ -184,8 +186,7 @@
    solved in 3.7 and perhaps in earlier versions too.) *)
 (* 32-bit hash, so we expect no collisions. *)
 fun controlled_length dfg s =
-  if dfg andalso size s > 60 then Word.toString (hashw_string (s, 0w0))
-  else s;
+  if dfg andalso size s > 60 then Word.toString (hashw_string (s, 0w0)) else s;
 
 fun lookup_const dfg c =
     case Symtab.lookup const_trans_table c of