src/Doc/Isar_Ref/Spec.thy
changeset 69913 ca515cf61651
parent 69597 ff784d5a5bfb
child 69962 82e945d472d5
--- a/src/Doc/Isar_Ref/Spec.thy	Thu Mar 14 16:35:58 2019 +0100
+++ b/src/Doc/Isar_Ref/Spec.thy	Thu Mar 14 16:55:06 2019 +0100
@@ -93,8 +93,8 @@
   proof documents work properly. Command keywords need to be classified
   according to their structural role in the formal text. Examples may be seen
   in Isabelle/HOL sources itself, such as @{keyword "keywords"}~\<^verbatim>\<open>"typedef"\<close>
-  \<open>:: thy_goal\<close> or @{keyword "keywords"}~\<^verbatim>\<open>"datatype"\<close> \<open>:: thy_decl\<close> for
-  theory-level declarations with and without proof, respectively. Additional
+  \<open>:: thy_goal_defn\<close> or @{keyword "keywords"}~\<^verbatim>\<open>"datatype"\<close> \<open>:: thy_defn\<close> for
+  theory-level definitions with and without proof, respectively. Additional
   @{syntax tags} provide defaults for document preparation
   (\secref{sec:tags}).