cosmetics
authorblanchet
Wed, 25 Aug 2010 09:34:28 +0200
changeset 38742 4fe1bb9e7434
parent 38741 7635bf8918a1
child 38743 69fa75354c58
cosmetics
src/HOL/Tools/Sledgehammer/sledgehammer_fact_filter.ML
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_fact_filter.ML	Wed Aug 25 09:32:43 2010 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_fact_filter.ML	Wed Aug 25 09:34:28 2010 +0200
@@ -244,11 +244,9 @@
   in if Real.isFinite res then res else 0.0 end
 *)
 
-(* Multiplies out to a list of pairs: 'a * 'b list -> ('a * 'b) list
-   -> ('a * 'b) list. *)
-fun add_expand_pairs (x, ys) xys = List.foldl (fn (y,acc) => (x,y)::acc) xys ys
 fun consts_of_term thy t =
-  Symtab.fold add_expand_pairs (get_consts thy (SOME true) [t]) []
+  Symtab.fold (fn (x, ys) => fold (fn y => cons (x, y)) ys)
+              (get_consts thy (SOME true) [t]) []
 
 fun pair_consts_axiom theory_relevant thy axiom =
   (axiom, axiom |> snd |> theory_const_prop_of theory_relevant