src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML
changeset 44599 d34ff13371e0
parent 44597 03bbadb252db
child 44634 2ac4ff398bc3
equal deleted inserted replaced
44598:b054ca3f07b5 44599:d34ff13371e0
   154 
   154 
   155 fun is_atp_for_format is_format ctxt name =
   155 fun is_atp_for_format is_format ctxt name =
   156   let val thy = Proof_Context.theory_of ctxt in
   156   let val thy = Proof_Context.theory_of ctxt in
   157     case try (get_atp thy) name of
   157     case try (get_atp thy) name of
   158       SOME {best_slices, ...} =>
   158       SOME {best_slices, ...} =>
   159       exists (fn (_, (_, (_, format, _, _))) => format = CNF_UEQ)
   159       exists (fn (_, (_, (_, format, _, _))) => is_format format)
   160              (best_slices ctxt)
   160              (best_slices ctxt)
   161     | NONE => false
   161     | NONE => false
   162   end
   162   end
   163 
   163 
   164 val is_unit_equational_atp = is_atp_for_format (curry (op =) CNF_UEQ)
   164 val is_unit_equational_atp = is_atp_for_format (curry (op =) CNF_UEQ)