src/HOL/Tools/Sledgehammer/sledgehammer_prover.ML
changeset 63692 1bc4bc2c9fd1
parent 62735 23de054397e5
child 71931 0c8a9c028304
equal deleted inserted replaced
63691:94a89b95b871 63692:1bc4bc2c9fd1
   192     val thy = Proof_Context.theory_of ctxt
   192     val thy = Proof_Context.theory_of ctxt
   193     val (remote_provers, local_provers) =
   193     val (remote_provers, local_provers) =
   194       sort_strings (supported_atps thy) @ sort_strings (SMT_Config.available_solvers_of ctxt)
   194       sort_strings (supported_atps thy) @ sort_strings (SMT_Config.available_solvers_of ctxt)
   195       |> List.partition (String.isPrefix remote_prefix)
   195       |> List.partition (String.isPrefix remote_prefix)
   196   in
   196   in
   197     writeln ("Supported provers: " ^ commas (local_provers @ remote_provers) ^ ".")
   197     writeln ("Supported provers: " ^ commas (local_provers @ remote_provers))
   198   end
   198   end
   199 
   199 
   200 end;
   200 end;