src/Doc/Isar_Ref/Document_Preparation.thy
changeset 73769 08db0a06e131
parent 73765 ebaed09ce06e
child 74122 7d3e818fe21f
equal deleted inserted replaced
73768:c73c22c62d08 73769:08db0a06e131
   204       @@{antiquotation prf} options @{syntax thms} |
   204       @@{antiquotation prf} options @{syntax thms} |
   205       @@{antiquotation full_prf} options @{syntax thms} |
   205       @@{antiquotation full_prf} options @{syntax thms} |
   206       @@{antiquotation ML_text} options @{syntax text} |
   206       @@{antiquotation ML_text} options @{syntax text} |
   207       @@{antiquotation ML} options @{syntax text} |
   207       @@{antiquotation ML} options @{syntax text} |
   208       @@{antiquotation ML_infix} options @{syntax text} |
   208       @@{antiquotation ML_infix} options @{syntax text} |
   209       @@{antiquotation ML_type} options @{syntax text} |
   209       @@{antiquotation ML_type} options @{syntax typeargs} @{syntax text} |
   210       @@{antiquotation ML_structure} options @{syntax text} |
   210       @@{antiquotation ML_structure} options @{syntax text} |
   211       @@{antiquotation ML_functor} options @{syntax text} |
   211       @@{antiquotation ML_functor} options @{syntax text} |
   212       @@{antiquotation emph} options @{syntax text} |
   212       @@{antiquotation emph} options @{syntax text} |
   213       @@{antiquotation bold} options @{syntax text} |
   213       @@{antiquotation bold} options @{syntax text} |
   214       @@{antiquotation verbatim} options @{syntax text} |
   214       @@{antiquotation verbatim} options @{syntax text} |
   300   \<open>@{ML_functor s}\<close> check text \<open>s\<close> as ML value, infix operator, type,
   300   \<open>@{ML_functor s}\<close> check text \<open>s\<close> as ML value, infix operator, type,
   301   exception, structure, and functor respectively. The source is printed
   301   exception, structure, and functor respectively. The source is printed
   302   verbatim. The variants \<open>@{ML_def s}\<close> and \<open>@{ML_ref s}\<close> etc. maintain the
   302   verbatim. The variants \<open>@{ML_def s}\<close> and \<open>@{ML_ref s}\<close> etc. maintain the
   303   document index: ``def'' means to make a bold entry, ``ref'' means to make a
   303   document index: ``def'' means to make a bold entry, ``ref'' means to make a
   304   regular entry.
   304   regular entry.
       
   305 
       
   306   There are two forms for type constructors, with or without separate type
       
   307   arguments: this impacts only the index entry. For example, \<open>@{ML_type_ref
       
   308   \<open>'a list\<close>}\<close> makes an entry literally for ``\<open>'a list\<close>'' (sorted under the
       
   309   letter ``a''), but \<open>@{ML_type_ref 'a \<open>list\<close>}\<close> makes an entry for the
       
   310   constructor name ``\<open>list\<close>''.
   305 
   311 
   306   \<^descr> \<open>@{emph s}\<close> prints document source recursively, with {\LaTeX} markup
   312   \<^descr> \<open>@{emph s}\<close> prints document source recursively, with {\LaTeX} markup
   307   \<^verbatim>\<open>\emph{\<close>\<open>\<dots>\<close>\<^verbatim>\<open>}\<close>.
   313   \<^verbatim>\<open>\emph{\<close>\<open>\<dots>\<close>\<^verbatim>\<open>}\<close>.
   308 
   314 
   309   \<^descr> \<open>@{bold s}\<close> prints document source recursively, with {\LaTeX} markup
   315   \<^descr> \<open>@{bold s}\<close> prints document source recursively, with {\LaTeX} markup