src/HOL/TPTP/atp_problem_import.ML
changeset 62718 27333dc58e28
parent 62519 a564458f94db
child 64445 233a11ed2dfb
equal deleted inserted replaced
62717:8adf274f5988 62718:27333dc58e28
   183 fun atp_tac ctxt completeness override_params timeout assms prover =
   183 fun atp_tac ctxt completeness override_params timeout assms prover =
   184   let
   184   let
   185     val thy = Proof_Context.theory_of ctxt
   185     val thy = Proof_Context.theory_of ctxt
   186     val assm_ths0 = map (Skip_Proof.make_thm thy) assms
   186     val assm_ths0 = map (Skip_Proof.make_thm thy) assms
   187     val ((assm_name, _), ctxt) = ctxt
   187     val ((assm_name, _), ctxt) = ctxt
   188       |> Config.put Sledgehammer_Prover_ATP.atp_completish (completeness > 0)
   188       |> Config.put Sledgehammer_Prover_ATP.atp_completish (if completeness > 0 then 2 else 0)
   189       |> Local_Theory.note ((@{binding thms}, []), assm_ths0)
   189       |> Local_Theory.note ((@{binding thms}, []), assm_ths0)
   190 
   190 
   191     fun ref_of th = (Facts.named (Thm.derivation_name th), [])
   191     fun ref_of th = (Facts.named (Thm.derivation_name th), [])
   192     val ref_of_assms = (Facts.named assm_name, [])
   192     val ref_of_assms = (Facts.named assm_name, [])
   193   in
   193   in