src/HOL/Tools/Sledgehammer/sledgehammer_commands.ML
changeset 74352 fb8ce6090437
parent 73940 f58108b7a60c
child 74369 3301c0d8b560
equal deleted inserted replaced
74351:d8dbe7525ff1 74352:fb8ce6090437
   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] @
   180   [cvc4N, vampireN, z3N, eN, spassN, veritN]
   181   (if is_vampire_noncommercial_license_accepted () = SOME false then [] else [vampireN]) @
       
   182   [z3N, eN, spassN, veritN]
       
   183   |> map_filter (remotify_prover_if_not_installed ctxt)
   181   |> map_filter (remotify_prover_if_not_installed ctxt)
   184   (* 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) *)
   185   |> take (Multithreading.max_threads () - (if mode = Try then 1 else 0))
   183   |> take (Multithreading.max_threads () - (if mode = Try then 1 else 0))
   186   |> implode_param
   184   |> implode_param
   187 
   185