src/HOL/Tools/Sledgehammer/sledgehammer_prover_minimize.ML
changeset 75024 114eb0af123d
parent 75023 fdda7e754f45
child 75025 f741d55a81e5
equal deleted inserted replaced
75023:fdda7e754f45 75024:114eb0af123d
    52   is_smt_prover ctxt orf is_atp_installed (Proof_Context.theory_of ctxt)
    52   is_smt_prover ctxt orf is_atp_installed (Proof_Context.theory_of ctxt)
    53 
    53 
    54 fun default_max_facts_of_prover ctxt name =
    54 fun default_max_facts_of_prover ctxt name =
    55   let val thy = Proof_Context.theory_of ctxt in
    55   let val thy = Proof_Context.theory_of ctxt in
    56     if is_atp thy name then
    56     if is_atp thy name then
    57       fold (Integer.max o fst o #1 o fst o snd) (#best_slices (get_atp thy name ()) ctxt) 0
    57       fold (Integer.max o fst o #1) (#best_slices (get_atp thy name ()) ctxt) 0
    58     else if is_smt_prover ctxt name then
    58     else if is_smt_prover ctxt name then
    59       SMT_Solver.default_max_relevant ctxt name
    59       SMT_Solver.default_max_relevant ctxt name
    60     else
    60     else
    61       error ("No such prover: " ^ name)
    61       error ("No such prover: " ^ name)
    62   end
    62   end