src/HOL/Tools/Sledgehammer/sledgehammer.ML
changeset 40562 bbcb7aa90afc
parent 40561 0125cbb5d3c7
parent 40559 9597b93a8c00
child 40627 becf5d5187cc
equal deleted inserted replaced
40561:0125cbb5d3c7 40562:bbcb7aa90afc
   514       | SOME SMT_Failure.Time_Out => "Timed out."
   514       | SOME SMT_Failure.Time_Out => "Timed out."
   515       | SOME (SMT_Failure.Abnormal_Termination code) =>
   515       | SOME (SMT_Failure.Abnormal_Termination code) =>
   516         "The SMT solver terminated abnormally with exit code " ^
   516         "The SMT solver terminated abnormally with exit code " ^
   517         string_of_int code ^ "."
   517         string_of_int code ^ "."
   518       | SOME (SMT_Failure.Counterexample _) => "The SMT problem is unprovable."
   518       | SOME (SMT_Failure.Counterexample _) => "The SMT problem is unprovable."
       
   519       | SOME SMT_Failure.Out_Of_Memory => "The SMT solver ran out of memory."
   519       | SOME failure =>
   520       | SOME failure =>
   520         SMT_Failure.string_of_failure ctxt failure
   521         SMT_Failure.string_of_failure ctxt failure
   521     val outcome = outcome |> Option.map failure_from_smt_failure (* FIXME *)
   522     val outcome = outcome |> Option.map failure_from_smt_failure (* FIXME *)
   522   in
   523   in
   523     {outcome = outcome, used_facts = used_facts,
   524     {outcome = outcome, used_facts = used_facts,