src/HOL/Mirabelle/Tools/mirabelle_sledgehammer.ML
changeset 39377 9e544eb396dc
parent 39366 f58fbb959826
child 39494 bf7dd4902321
equal deleted inserted replaced
39376:ca81b7ae543c 39377:9e544eb396dc
   403     val (msg, result) = run_sh prover_name prover hard_timeout timeout dir st
   403     val (msg, result) = run_sh prover_name prover hard_timeout timeout dir st
   404   in
   404   in
   405     case result of
   405     case result of
   406       SH_OK (time_isa, time_atp, names) =>
   406       SH_OK (time_isa, time_atp, names) =>
   407         let
   407         let
   408           fun get_thms (name, Sledgehammer_Filter.Chained) = NONE
   408           fun get_thms (_, Sledgehammer_Filter.Chained) = NONE
   409             | get_thms (name, loc) =
   409             | get_thms (name, loc) =
   410               SOME ((name, loc), thms_of_name (Proof.context_of st) name)
   410               SOME ((name, loc), thms_of_name (Proof.context_of st) name)
   411         in
   411         in
   412           change_data id inc_sh_success;
   412           change_data id inc_sh_success;
   413           if trivial then () else change_data id inc_sh_nontriv_success;
   413           if trivial then () else change_data id inc_sh_nontriv_success;