src/Pure/Isar/induct_attrib.ML
changeset 18728 6790126ab5f6
parent 18708 4b3dadb4fe33
child 18977 f24c416a4814
equal deleted inserted replaced
18727:caf9bc780c80 18728:6790126ab5f6
    23   val find_casesS: Proof.context -> term -> thm list
    23   val find_casesS: Proof.context -> term -> thm list
    24   val find_inductT: Proof.context -> typ -> thm list
    24   val find_inductT: Proof.context -> typ -> thm list
    25   val find_inductS: Proof.context -> term -> thm list
    25   val find_inductS: Proof.context -> term -> thm list
    26   val find_coinductT: Proof.context -> typ -> thm list
    26   val find_coinductT: Proof.context -> typ -> thm list
    27   val find_coinductS: Proof.context -> term -> thm list
    27   val find_coinductS: Proof.context -> term -> thm list
    28   val cases_type: string -> Context.generic attribute
    28   val cases_type: string -> attribute
    29   val cases_set: string -> Context.generic attribute
    29   val cases_set: string -> attribute
    30   val induct_type: string -> Context.generic attribute
    30   val induct_type: string -> attribute
    31   val induct_set: string -> Context.generic attribute
    31   val induct_set: string -> attribute
    32   val coinduct_type: string -> Context.generic attribute
    32   val coinduct_type: string -> attribute
    33   val coinduct_set: string -> Context.generic attribute
    33   val coinduct_set: string -> attribute
    34   val casesN: string
    34   val casesN: string
    35   val inductN: string
    35   val inductN: string
    36   val coinductN: string
    36   val coinductN: string
    37   val typeN: string
    37   val typeN: string
    38   val setN: string
    38   val setN: string
   223 
   223 
   224 end;
   224 end;
   225 
   225 
   226 val _ = Context.add_setup
   226 val _ = Context.add_setup
   227  (Attrib.add_attributes
   227  (Attrib.add_attributes
   228   [(casesN, Attrib.common cases_att, "declaration of cases rule for type or set"),
   228   [(casesN, cases_att, "declaration of cases rule for type or set"),
   229    (inductN, Attrib.common induct_att, "declaration of induction rule for type or set"),
   229    (inductN, induct_att, "declaration of induction rule for type or set"),
   230    (coinductN, Attrib.common coinduct_att, "declaration of coinduction rule for type or set")]);
   230    (coinductN, coinduct_att, "declaration of coinduction rule for type or set")]);
   231 
   231 
   232 end;
   232 end;