src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML
changeset 41126 e0bd443c0fdd
parent 41103 eaefbe8aac1c
child 41134 de9e0adc21da
equal deleted inserted replaced
41125:4a9eec045f2a 41126:e0bd443c0fdd
   526       Context.proof_map (SMT_Config.select_solver suffix)
   526       Context.proof_map (SMT_Config.select_solver suffix)
   527       #> Config.put SMT_Config.verbose debug
   527       #> Config.put SMT_Config.verbose debug
   528       #> Config.put SMT_Config.monomorph_limit smt_monomorph_limit
   528       #> Config.put SMT_Config.monomorph_limit smt_monomorph_limit
   529     val state = state |> Proof.map_context repair_context
   529     val state = state |> Proof.map_context repair_context
   530     val thy = Proof.theory_of state
   530     val thy = Proof.theory_of state
   531     val facts = facts |> map (apsnd (Thm.transfer thy) o untranslated_fact)
   531     val facts = facts |> map (apsnd (pair NONE o Thm.transfer thy) o untranslated_fact)
   532     val {outcome, used_facts, run_time_in_msecs} =
   532     val {outcome, used_facts, run_time_in_msecs} =
   533       smt_filter_loop params remote state subgoal facts
   533       smt_filter_loop params remote state subgoal facts
   534     val (chained_lemmas, other_lemmas) = split_used_facts (map fst used_facts)
   534     val (chained_lemmas, other_lemmas) = split_used_facts (map fst used_facts)
   535     val outcome = outcome |> Option.map failure_from_smt_failure
   535     val outcome = outcome |> Option.map failure_from_smt_failure
   536     val message =
   536     val message =