src/HOL/TPTP/TPTP_Proof_Reconstruction.thy
changeset 57773 2719eb9d40fe
parent 56252 b72e0a9d62b9
child 58411 e3d0354d2129
equal deleted inserted replaced
57772:7d9134b032b2 57773:2719eb9d40fe
  2114         | SOME {inference_name, ...} => inference_name
  2114         | SOME {inference_name, ...} => inference_name
  2115     val default_tac = HEADGOAL (blast_tac ctxt)
  2115     val default_tac = HEADGOAL (blast_tac ctxt)
  2116   in
  2116   in
  2117     case inference_name of
  2117     case inference_name of
  2118       "fo_atp_e" =>
  2118       "fo_atp_e" =>
       
  2119         HEADGOAL (Metis_Tactic.metis_tac [] ATP_Problem_Generate.combs_or_liftingN ctxt [])
       
  2120         (*NOTE To treat E as an oracle use the following line:
  2119         HEADGOAL (etac (oracle_based_reconstruction_tac ctxt prob_name node))
  2121         HEADGOAL (etac (oracle_based_reconstruction_tac ctxt prob_name node))
       
  2122         *)
  2120     | "copy" =>
  2123     | "copy" =>
  2121          HEADGOAL
  2124          HEADGOAL
  2122           (atac
  2125           (atac
  2123            ORELSE'
  2126            ORELSE'
  2124               (rtac @{thm polarise}
  2127               (rtac @{thm polarise}