src/HOL/Tools/Sledgehammer/sledgehammer_run.ML
changeset 53804 58d1b63bea81
parent 53800 ac1ec5065316
child 53814 255a2929c137
equal deleted inserted replaced
53803:b6a947a2c615 53804:58d1b63bea81
   223       val _ = () |> not blocking ? kill_provers
   223       val _ = () |> not blocking ? kill_provers
   224       val _ = case find_first (not o is_prover_supported ctxt) provers of
   224       val _ = case find_first (not o is_prover_supported ctxt) provers of
   225                 SOME name => error ("No such prover: " ^ name ^ ".")
   225                 SOME name => error ("No such prover: " ^ name ^ ".")
   226               | NONE => ()
   226               | NONE => ()
   227       val _ = print "Sledgehammering..."
   227       val _ = print "Sledgehammering..."
   228       val _ = spying spy (fn () => ("***", "run"))
   228       val _ = spying spy (fn () => ("***", "starting " ^ @{make_string} mode ^ " mode"))
   229       val (smts, (ueq_atps, full_atps)) =
   229       val (smts, (ueq_atps, full_atps)) =
   230         provers |> List.partition (is_smt_prover ctxt)
   230         provers |> List.partition (is_smt_prover ctxt)
   231                 ||> List.partition (is_unit_equational_atp ctxt)
   231                 ||> List.partition (is_unit_equational_atp ctxt)
   232 
   232 
   233       val spying_str_of_factss =
   233       val spying_str_of_factss =