src/Pure/Isar/induct_attrib.ML
changeset 21506 b2a673894ce5
parent 19046 bc5c6c9b114e
child 22360 26ead7ed4f4b
--- a/src/Pure/Isar/induct_attrib.ML	Thu Nov 23 22:38:29 2006 +0100
+++ b/src/Pure/Isar/induct_attrib.ML	Thu Nov 23 22:38:30 2006 +0100
@@ -8,11 +8,11 @@
 signature INDUCT_ATTRIB =
 sig
   val vars_of: term -> term list
-  val dest_rules: Context.generic ->
+  val dest_rules: Proof.context ->
     {type_cases: (string * thm) list, set_cases: (string * thm) list,
       type_induct: (string * thm) list, set_induct: (string * thm) list,
       type_coinduct: (string * thm) list, set_coinduct: (string * thm) list}
-  val print_rules: Context.generic -> unit
+  val print_rules: Proof.context -> unit
   val lookup_casesT : Proof.context -> string -> thm option
   val lookup_casesS : Proof.context -> string -> thm option
   val lookup_inductT : Proof.context -> string -> thm option
@@ -133,8 +133,8 @@
 );
 
 val _ = Context.add_setup Induct.init;
-val print_rules = Induct.print;
-val dest_rules = dest o Induct.get;
+val print_rules = Induct.print o Context.Proof;
+val dest_rules = dest o Induct.get o Context.Proof;
 
 val get_local = Induct.get o Context.Proof;