src/HOL/BNF/BNF_GFP.thy
changeset 53822 6304b12c7627
parent 53753 ae7f50e70c09
child 54246 8fdb4dc08ed1
--- a/src/HOL/BNF/BNF_GFP.thy	Tue Sep 24 14:07:23 2013 +0200
+++ b/src/HOL/BNF/BNF_GFP.thy	Tue Sep 24 15:16:59 2013 +0200
@@ -11,7 +11,8 @@
 imports BNF_FP_Base Equiv_Relations_More "~~/src/HOL/Library/Sublist"
 keywords
   "codatatype" :: thy_decl and
-  "primcorecursive" :: thy_goal
+  "primcorecursive" :: thy_goal and
+  "primcorec" :: thy_decl
 begin
 
 lemma sum_case_expand_Inr: "f o Inl = g \<Longrightarrow> f x = sum_case g (f o Inr) x"