src/HOL/Tools/Sledgehammer/sledgehammer_translate.ML
changeset 40059 6ad9081665db
parent 39975 7c50d5ca5c04
equal deleted inserted replaced
40058:b4f62d0660e0 40059:6ad9081665db
    14   val axiom_prefix : string
    14   val axiom_prefix : string
    15   val conjecture_prefix : string
    15   val conjecture_prefix : string
    16   val prepare_axiom :
    16   val prepare_axiom :
    17     Proof.context -> (string * 'a) * thm
    17     Proof.context -> (string * 'a) * thm
    18     -> term * ((string * 'a) * fol_formula) option
    18     -> term * ((string * 'a) * fol_formula) option
    19   val prepare_problem :
    19   val prepare_atp_problem :
    20     Proof.context -> bool -> bool -> bool -> bool -> term list -> term
    20     Proof.context -> bool -> bool -> bool -> bool -> term list -> term
    21     -> (term * ((string * 'a) * fol_formula) option) list
    21     -> (term * ((string * 'a) * fol_formula) option) list
    22     -> string problem * string Symtab.table * int * (string * 'a) list vector
    22     -> string problem * string Symtab.table * int * (string * 'a) list vector
    23 end;
    23 end;
    24 
    24 
   492 
   492 
   493 fun repair_problem thy explicit_forall full_types explicit_apply problem =
   493 fun repair_problem thy explicit_forall full_types explicit_apply problem =
   494   repair_problem_with_const_table thy explicit_forall full_types
   494   repair_problem_with_const_table thy explicit_forall full_types
   495       (const_table_for_problem explicit_apply problem) problem
   495       (const_table_for_problem explicit_apply problem) problem
   496 
   496 
   497 fun prepare_problem ctxt readable_names explicit_forall full_types
   497 fun prepare_atp_problem ctxt readable_names explicit_forall full_types
   498                     explicit_apply hyp_ts concl_t axioms =
   498                         explicit_apply hyp_ts concl_t axioms =
   499   let
   499   let
   500     val thy = ProofContext.theory_of ctxt
   500     val thy = ProofContext.theory_of ctxt
   501     val (axiom_names, (conjectures, axioms, helper_facts, class_rel_clauses,
   501     val (axiom_names, (conjectures, axioms, helper_facts, class_rel_clauses,
   502                        arity_clauses)) =
   502                        arity_clauses)) =
   503       prepare_formulas ctxt full_types hyp_ts concl_t axioms
   503       prepare_formulas ctxt full_types hyp_ts concl_t axioms