src/HOL/Tools/Sledgehammer/sledgehammer_prover_atp.ML
changeset 57460 9cc802a8ab06
parent 57267 8b87114357bd
child 57671 dc5e1b1db9ba
equal deleted inserted replaced
57459:22023ab4df3c 57460:9cc802a8ab06
   381                     val metis_lam_trans =
   381                     val metis_lam_trans =
   382                       if atp_proof_prefers_lifting atp_proof then SOME liftingN else NONE
   382                       if atp_proof_prefers_lifting atp_proof then SOME liftingN else NONE
   383                     val atp_proof =
   383                     val atp_proof =
   384                       atp_proof
   384                       atp_proof
   385                       |> termify_atp_proof ctxt name format type_enc pool lifted sym_tab
   385                       |> termify_atp_proof ctxt name format type_enc pool lifted sym_tab
   386                       |> introduce_spass_skolem
   386                       |> spass ? introduce_spass_skolem
   387                       |> factify_atp_proof (map fst used_from) hyp_ts concl_t
   387                       |> factify_atp_proof (map fst used_from) hyp_ts concl_t
   388                   in
   388                   in
   389                     (verbose, (metis_type_enc, metis_lam_trans), preplay_timeout, compress, try0,
   389                     (verbose, (metis_type_enc, metis_lam_trans), preplay_timeout, compress, try0,
   390                      minimize <> SOME false, atp_proof, goal)
   390                      minimize <> SOME false, atp_proof, goal)
   391                   end
   391                   end