src/HOL/Tools/Sledgehammer/sledgehammer_commands.ML
changeset 74822 4e30de0b4dd6
parent 74738 d8dc8fdc46fc
child 74894 3315c551fe6e
equal deleted inserted replaced
74821:4bb1251043cd 74822:4e30de0b4dd6
   175   if is_prover_supported ctxt name andalso is_prover_installed ctxt name then SOME name
   175   if is_prover_supported ctxt name andalso is_prover_installed ctxt name then SOME name
   176   else remotify_prover_if_supported_and_not_already_remote ctxt name
   176   else remotify_prover_if_supported_and_not_already_remote ctxt name
   177 
   177 
   178 (* The first ATP of the list is used by Auto Sledgehammer. *)
   178 (* The first ATP of the list is used by Auto Sledgehammer. *)
   179 fun default_provers_param_value mode ctxt =
   179 fun default_provers_param_value mode ctxt =
   180   [cvc4N, vampireN, veritN, eN, spassN, z3N, zipperpositionN]
   180   [cvc4N, vampireN, veritN, eN, spassN, z3N, zipperpositionN] \<comment> \<open>see also \<^system_option>\<open>sledgehammer_provers\<close>\<close>
   181   |> map_filter (remotify_prover_if_not_installed ctxt)
   181   |> map_filter (remotify_prover_if_not_installed ctxt)
   182   (* In "try" mode, leave at least one thread to another slow tool (e.g. Nitpick) *)
   182   (* In "try" mode, leave at least one thread to another slow tool (e.g. Nitpick) *)
   183   |> take (Multithreading.max_threads () - (if mode = Try then 1 else 0))
   183   |> take (Multithreading.max_threads () - (if mode = Try then 1 else 0))
   184   |> implode_param
   184   |> implode_param
   185 
   185