src/HOL/Nominal/Nominal.thy
changeset 69913 ca515cf61651
parent 69605 a96320074298
child 80129 601ff5c7cad5
--- a/src/HOL/Nominal/Nominal.thy	Thu Mar 14 16:35:58 2019 +0100
+++ b/src/HOL/Nominal/Nominal.thy	Thu Mar 14 16:55:06 2019 +0100
@@ -1,8 +1,10 @@
 theory Nominal 
 imports "HOL-Library.Infinite_Set" "HOL-Library.Old_Datatype"
 keywords
-  "atom_decl" "nominal_datatype" "equivariance" :: thy_decl and
-  "nominal_primrec" "nominal_inductive" "nominal_inductive2" :: thy_goal and
+  "atom_decl" :: thy_decl and
+  "nominal_datatype" :: thy_defn and
+  "equivariance" :: thy_decl and
+  "nominal_primrec" "nominal_inductive" "nominal_inductive2" :: thy_goal_defn and
   "avoids"
 begin