src/HOL/Codatatype/Tools/bnf_lfp.ML
changeset 49205 674f04c737e0
parent 49185 073d7d1b7488
child 49222 cbe8c859817c
--- a/src/HOL/Codatatype/Tools/bnf_lfp.ML	Sat Sep 08 21:04:26 2012 +0200
+++ b/src/HOL/Codatatype/Tools/bnf_lfp.ML	Sat Sep 08 21:04:26 2012 +0200
@@ -8,9 +8,10 @@
 
 signature BNF_LFP =
 sig
-  val bnf_lfp:  mixfix list -> (string * sort) list option -> binding list ->
+  val bnf_lfp: mixfix list -> (string * sort) list option -> binding list ->
     typ list * typ list list -> BNF_Def.BNF list -> local_theory ->
-    (term list * term list * term list * term list * thm list * thm list * thm list) * local_theory
+    (term list * term list * term list * term list * thm list * thm list * thm list * thm list *
+      thm list) * local_theory
 end;
 
 structure BNF_LFP : BNF_LFP =
@@ -1822,8 +1823,8 @@
             ((Binding.qualify true (Binding.name_of b) (Binding.name thmN), []), [(thms, [])]))
           bs thmss)
   in
-    ((unfs, flds, iters, recs, unf_fld_thms, fld_unf_thms, fld_inject_thms),
-      lthy |> Local_Theory.notes (common_notes @ notes) |> snd)
+    ((unfs, flds, iters, recs, unf_fld_thms, fld_unf_thms, fld_inject_thms, iter_thms, rec_thms),
+     lthy |> Local_Theory.notes (common_notes @ notes) |> snd)
   end;
 
 val _ =