src/Pure/Tools/rule_insts.ML
changeset 55151 f331472f1027
parent 55143 04448228381d
child 55156 3ca79ee6eb33
equal deleted inserted replaced
55150:0940309ed8f1 55151:f331472f1027
     4 Rule instantiations -- operations within implicit rule / subgoal context.
     4 Rule instantiations -- operations within implicit rule / subgoal context.
     5 *)
     5 *)
     6 
     6 
     7 signature BASIC_RULE_INSTS =
     7 signature BASIC_RULE_INSTS =
     8 sig
     8 sig
     9   val read_instantiate: Proof.context -> (indexname * string) list -> string list -> thm -> thm
       
    10   val instantiate_tac: Proof.context -> (indexname * string) list -> string list -> tactic
       
    11   val res_inst_tac: Proof.context -> (indexname * string) list -> thm -> int -> tactic
     9   val res_inst_tac: Proof.context -> (indexname * string) list -> thm -> int -> tactic
    12   val eres_inst_tac: Proof.context -> (indexname * string) list -> thm -> int -> tactic
    10   val eres_inst_tac: Proof.context -> (indexname * string) list -> thm -> int -> tactic
    13   val cut_inst_tac: Proof.context -> (indexname * string) list -> thm -> int -> tactic
    11   val cut_inst_tac: Proof.context -> (indexname * string) list -> thm -> int -> tactic
    14   val forw_inst_tac: Proof.context -> (indexname * string) list -> thm -> int -> tactic
    12   val forw_inst_tac: Proof.context -> (indexname * string) list -> thm -> int -> tactic
    15   val dres_inst_tac: Proof.context -> (indexname * string) list -> thm -> int -> tactic
    13   val dres_inst_tac: Proof.context -> (indexname * string) list -> thm -> int -> tactic
    22   include BASIC_RULE_INSTS
    20   include BASIC_RULE_INSTS
    23   val where_rule: Proof.context -> (indexname * string) list ->
    21   val where_rule: Proof.context -> (indexname * string) list ->
    24     (binding * string option * mixfix) list -> thm -> thm
    22     (binding * string option * mixfix) list -> thm -> thm
    25   val of_rule: Proof.context -> string option list * string option list ->
    23   val of_rule: Proof.context -> string option list * string option list ->
    26     (binding * string option * mixfix) list -> thm -> thm
    24     (binding * string option * mixfix) list -> thm -> thm
       
    25   val read_instantiate: Proof.context -> (indexname * string) list -> string list -> thm -> thm
       
    26   val instantiate_tac: Proof.context -> (indexname * string) list -> string list -> tactic
    27   val make_elim_preserve: thm -> thm
    27   val make_elim_preserve: thm -> thm
    28   val method: (Proof.context -> (indexname * string) list -> thm -> int -> tactic) ->
    28   val method: (Proof.context -> (indexname * string) list -> thm -> int -> tactic) ->
    29     (Proof.context -> thm list -> int -> tactic) -> (Proof.context -> Proof.method) context_parser
    29     (Proof.context -> thm list -> int -> tactic) -> (Proof.context -> Proof.method) context_parser
    30 end;
    30 end;
    31 
    31