src/HOL/Inductive.thy
changeset 69913 ca515cf61651
parent 69605 a96320074298
--- a/src/HOL/Inductive.thy	Thu Mar 14 16:35:58 2019 +0100
+++ b/src/HOL/Inductive.thy	Thu Mar 14 16:55:06 2019 +0100
@@ -7,11 +7,11 @@
 theory Inductive
   imports Complete_Lattices Ctr_Sugar
   keywords
-    "inductive" "coinductive" "inductive_cases" "inductive_simps" :: thy_decl and
+    "inductive" "coinductive" "inductive_cases" "inductive_simps" :: thy_defn and
     "monos" and
     "print_inductives" :: diag and
     "old_rep_datatype" :: thy_goal and
-    "primrec" :: thy_decl
+    "primrec" :: thy_defn
 begin
 
 subsection \<open>Least fixed points\<close>