--- a/src/HOL/Tools/Sledgehammer/sledgehammer_mepo.ML Sun Jan 28 16:09:00 2018 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_mepo.ML Sun Jan 28 19:28:52 2018 +0100
@@ -362,7 +362,7 @@
Math.pow (Real.fromInt remaining_max / Real.fromInt max_facts, max_imperfect_exp)))
val (perfect, imperfect) = candidates
|> sort (Real.compare o swap o apply2 snd)
- |> take_prefix (fn (_, w) => w > 0.99999)
+ |> chop_prefix (fn (_, w) => w > 0.99999)
val ((accepts, more_rejects), rejects) =
chop max_imperfect imperfect |>> append perfect |>> chop remaining_max
in