src/HOL/BNF_Least_Fixpoint.thy
changeset 69913 ca515cf61651
parent 69605 a96320074298
child 71836 c095d3143047
--- a/src/HOL/BNF_Least_Fixpoint.thy	Thu Mar 14 16:35:58 2019 +0100
+++ b/src/HOL/BNF_Least_Fixpoint.thy	Thu Mar 14 16:55:06 2019 +0100
@@ -12,8 +12,8 @@
 theory BNF_Least_Fixpoint
 imports BNF_Fixpoint_Base
 keywords
-  "datatype" :: thy_decl and
-  "datatype_compat" :: thy_decl
+  "datatype" :: thy_defn and
+  "datatype_compat" :: thy_defn
 begin
 
 lemma subset_emptyI: "(\<And>x. x \<in> A \<Longrightarrow> False) \<Longrightarrow> A \<subseteq> {}"