src/HOL/Tools/Metis/metis_tactics.ML
changeset 43135 8c32a0160b0d
parent 43134 0c82e00ba63e
child 43136 cf5cda219058
equal deleted inserted replaced
43134:0c82e00ba63e 43135:8c32a0160b0d
    57 fun used_axioms axioms (th, Metis_Proof.Axiom _) = SOME (lookth axioms th)
    57 fun used_axioms axioms (th, Metis_Proof.Axiom _) = SOME (lookth axioms th)
    58   | used_axioms _ _ = NONE
    58   | used_axioms _ _ = NONE
    59 
    59 
    60 fun cterm_from_metis ctxt sym_tab wrap tm =
    60 fun cterm_from_metis ctxt sym_tab wrap tm =
    61   let val thy = Proof_Context.theory_of ctxt in
    61   let val thy = Proof_Context.theory_of ctxt in
    62     tm |> hol_term_from_metis MX sym_tab ctxt
    62     tm |> hol_term_from_metis ctxt MX sym_tab |> wrap
    63        |> wrap
       
    64        |> Syntax.check_term
    63        |> Syntax.check_term
    65               (Proof_Context.set_mode Proof_Context.mode_schematic ctxt)
    64               (Proof_Context.set_mode Proof_Context.mode_schematic ctxt)
    66        |> cterm_of thy
    65        |> cterm_of thy
    67   end
    66   end
    68 
    67