src/HOL/Tools/Sledgehammer/sledgehammer_commands.ML
changeset 55458 d3b72d260d4a
parent 55297 1dfcd49f5dcb
child 55475 b8ebbcc5e49a
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_commands.ML	Thu Feb 13 15:51:54 2014 +0100
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_commands.ML	Thu Feb 13 16:21:43 2014 +0100
@@ -197,7 +197,7 @@
 (* The first ATP of the list is used by Auto Sledgehammer. Because of the low
    timeout, it makes sense to put E first. *)
 fun default_provers_param_value mode thy =
-  [eN, spassN, z3N, vampireN, e_sineN, yicesN]
+  [eN, spassN, z3N, e_sineN, vampireN, yicesN]
   |> map_filter (remotify_atp_if_not_installed thy)
   (* In "try" mode, leave at least one thread to another slow tool (e.g. Nitpick) *)
   |> take (Multithreading.max_threads_value () - (if mode = Try then 1 else 0))