src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML
changeset 40359 e5ed638e49b0
parent 40253 27f2a45b0aab
child 40385 c0da8252b2fa
     1.1 --- a/src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML	Fri Oct 22 18:31:45 2010 +0200
     1.2 +++ b/src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML	Mon Oct 25 09:29:43 2010 +0200
     1.3 @@ -157,13 +157,15 @@
     1.4        prover :: avoid_too_many_local_threads thy n provers
     1.5      end
     1.6  
     1.7 +val num_processors = try Thread.numProcessors #> the_default 1
     1.8 +
     1.9  (* The first ATP of the list is used by Auto Sledgehammer. Because of the low
    1.10     timeout, it makes sense to put SPASS first. *)
    1.11  fun default_provers_param_value ctxt =
    1.12    let val thy = ProofContext.theory_of ctxt in
    1.13      [spassN, eN, vampireN, sine_eN (* FIXME: , smtN *)]
    1.14      |> map_filter (remotify_prover_if_not_installed ctxt)
    1.15 -    |> avoid_too_many_local_threads thy (Thread.numProcessors ())
    1.16 +    |> avoid_too_many_local_threads thy (num_processors ())
    1.17      |> space_implode " "
    1.18    end
    1.19