src/HOL/BNF/BNF_GFP.thy
changeset 51804 be6e703908f4
parent 51782 84e7225f5ab6
child 51850 106afdf5806c
--- a/src/HOL/BNF/BNF_GFP.thy	Mon Apr 29 06:13:36 2013 +0200
+++ b/src/HOL/BNF/BNF_GFP.thy	Mon Apr 29 09:10:49 2013 +0200
@@ -10,7 +10,7 @@
 theory BNF_GFP
 imports BNF_FP Equiv_Relations_More "~~/src/HOL/Library/Sublist"
 keywords
-  "codata" :: thy_decl
+  "codatatype" :: thy_decl
 begin
 
 lemma o_sum_case: "h o sum_case f g = sum_case (h o f) (h o g)"