src/HOL/Tools/function_package/inductive_wrap.ML
changeset 22166 0a50d4db234a
parent 21365 4ee8e2702241
child 22612 1f017e6a0395
--- a/src/HOL/Tools/function_package/inductive_wrap.ML	Mon Jan 22 16:53:33 2007 +0100
+++ b/src/HOL/Tools/function_package/inductive_wrap.ML	Mon Jan 22 17:29:43 2007 +0100
@@ -11,7 +11,7 @@
 sig
   val inductive_def :  term list 
                        -> ((bstring * typ) * mixfix) * local_theory
-                       -> thm list * (term * thm * local_theory)
+                       -> thm list * (term * thm * thm * local_theory)
 end
 
 structure FundefInductiveWrap =
@@ -40,7 +40,7 @@
     let
       val qdefs = map dest_all_all defs
                   
-      val ({intrs = intrs_gen, elims = [elim_gen], preds = [ Rdef ], ...}, lthy) =
+      val ({intrs = intrs_gen, elims = [elim_gen], preds = [ Rdef ], induct, ...}, lthy) =
           InductivePackage.add_inductive_i true (*verbose*)
                                            "" (* no altname *)
                                            false (* no coind *)
@@ -70,7 +70,7 @@
                        |> Term.strip_comb |> snd |> hd (* Trueprop *)
                        |> Term.strip_comb |> fst
     in
-      (intrs, (Rdef_real, elim, lthy))
+      (intrs, (Rdef_real, elim, induct, lthy))
     end
     
 end