src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML
changeset 48513 9a9218111085
parent 47934 101976132929
child 48977 137883567114
     1.1 --- a/src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML	Sat Apr 21 07:33:47 2012 +0200
     1.2 +++ b/src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML	Sat Apr 21 11:15:49 2012 +0200
     1.3 @@ -215,7 +215,7 @@
     1.4  (* The first ATP of the list is used by Auto Sledgehammer. Because of the low
     1.5     timeout, it makes sense to put SPASS first. *)
     1.6  fun default_provers_param_value ctxt =
     1.7 -  [spassN, eN, vampireN, SMT_Solver.solver_name_of ctxt, satallaxN,
     1.8 +  [spassN, eN, vampireN, SMT_Solver.solver_name_of ctxt, e_sineN,
     1.9     waldmeisterN]
    1.10    |> map_filter (remotify_prover_if_not_installed ctxt)
    1.11    |> avoid_too_many_threads ctxt (Multithreading.max_threads_value (),