src/HOL/Tools/Nitpick/nitpick_util.ML
changeset 61770 a20048c78891
parent 59582 0fbed69ff081
child 61877 276ad4354069
equal deleted inserted replaced
61769:2cd36f4c5d65 61770:a20048c78891
    63   val instantiate_type : theory -> typ -> typ -> typ -> typ
    63   val instantiate_type : theory -> typ -> typ -> typ -> typ
    64   val varify_and_instantiate_type : Proof.context -> typ -> typ -> typ -> typ
    64   val varify_and_instantiate_type : Proof.context -> typ -> typ -> typ -> typ
    65   val varify_and_instantiate_type_global : theory -> typ -> typ -> typ -> typ
    65   val varify_and_instantiate_type_global : theory -> typ -> typ -> typ -> typ
    66   val is_of_class_const : theory -> string * typ -> bool
    66   val is_of_class_const : theory -> string * typ -> bool
    67   val get_class_def : theory -> string -> (string * term) option
    67   val get_class_def : theory -> string -> (string * term) option
    68   val monomorphic_term : Type.tyenv -> term -> term
       
    69   val specialize_type : theory -> string * typ -> term -> term
    68   val specialize_type : theory -> string * typ -> term -> term
    70   val eta_expand : typ list -> term -> int -> term
    69   val eta_expand : typ list -> term -> int -> term
    71   val DETERM_TIMEOUT : Time.time -> tactic -> tactic
    70   val DETERM_TIMEOUT : Time.time -> tactic -> tactic
    72   val indent_size : int
    71   val indent_size : int
    73   val pretty_maybe_quote : Keyword.keywords -> Pretty.T -> Pretty.T
    72   val pretty_maybe_quote : Keyword.keywords -> Pretty.T -> Pretty.T
   268   let val axname = class ^ "_class_def" in
   267   let val axname = class ^ "_class_def" in
   269     Option.map (pair axname)
   268     Option.map (pair axname)
   270       (AList.lookup (op =) (Theory.all_axioms_of thy) axname)
   269       (AList.lookup (op =) (Theory.all_axioms_of thy) axname)
   271   end;
   270   end;
   272 
   271 
   273 val monomorphic_term = ATP_Util.monomorphic_term
       
   274 val specialize_type = ATP_Util.specialize_type
   272 val specialize_type = ATP_Util.specialize_type
   275 val eta_expand = ATP_Util.eta_expand
   273 val eta_expand = ATP_Util.eta_expand
   276 
   274 
   277 fun DETERM_TIMEOUT delay tac st =
   275 fun DETERM_TIMEOUT delay tac st =
   278   Seq.of_list (the_list (TimeLimit.timeLimit delay (fn () => SINGLE tac st) ()))
   276   Seq.of_list (the_list (TimeLimit.timeLimit delay (fn () => SINGLE tac st) ()))