src/HOL/Nominal/nominal_induct.ML
changeset 61834 2154e6c8d52d
parent 61424 c3658c18b7bc
child 61841 4d3527b94f2a
equal deleted inserted replaced
61830:4f5ab843cf5b 61834:2154e6c8d52d
     5 
     5 
     6 structure NominalInduct:
     6 structure NominalInduct:
     7 sig
     7 sig
     8   val nominal_induct_tac: Proof.context -> bool -> (binding option * (term * bool)) option list list ->
     8   val nominal_induct_tac: Proof.context -> bool -> (binding option * (term * bool)) option list list ->
     9     (string * typ) list -> (string * typ) list list -> thm list ->
     9     (string * typ) list -> (string * typ) list list -> thm list ->
    10     thm list -> int -> Rule_Cases.cases_tactic
    10     thm list -> int -> cases_tactic
    11   val nominal_induct_method: (Proof.context -> Proof.method) context_parser
    11   val nominal_induct_method: (Proof.context -> Proof.method) context_parser
    12 end =
    12 end =
    13 struct
    13 struct
    14 
    14 
    15 (* proper tuples -- nested left *)
    15 (* proper tuples -- nested left *)