src/Doc/Isar_Ref/Document_Preparation.thy
changeset 71146 f7a9889068ff
parent 70140 d13865c21e36
child 71902 1529336eaedc
equal deleted inserted replaced
71145:2f782d5f5d5a 71146:f7a9889068ff
   106     @{antiquotation_def ML_structure} & : & \<open>antiquotation\<close> \\
   106     @{antiquotation_def ML_structure} & : & \<open>antiquotation\<close> \\
   107     @{antiquotation_def ML_functor} & : & \<open>antiquotation\<close> \\
   107     @{antiquotation_def ML_functor} & : & \<open>antiquotation\<close> \\
   108     @{antiquotation_def emph} & : & \<open>antiquotation\<close> \\
   108     @{antiquotation_def emph} & : & \<open>antiquotation\<close> \\
   109     @{antiquotation_def bold} & : & \<open>antiquotation\<close> \\
   109     @{antiquotation_def bold} & : & \<open>antiquotation\<close> \\
   110     @{antiquotation_def verbatim} & : & \<open>antiquotation\<close> \\
   110     @{antiquotation_def verbatim} & : & \<open>antiquotation\<close> \\
       
   111     @{antiquotation_def system_option} & : & \<open>antiquotation\<close> \\
   111     @{antiquotation_def session} & : & \<open>antiquotation\<close> \\
   112     @{antiquotation_def session} & : & \<open>antiquotation\<close> \\
   112     @{antiquotation_def "file"} & : & \<open>antiquotation\<close> \\
   113     @{antiquotation_def "file"} & : & \<open>antiquotation\<close> \\
   113     @{antiquotation_def "url"} & : & \<open>antiquotation\<close> \\
   114     @{antiquotation_def "url"} & : & \<open>antiquotation\<close> \\
   114     @{antiquotation_def "cite"} & : & \<open>antiquotation\<close> \\
   115     @{antiquotation_def "cite"} & : & \<open>antiquotation\<close> \\
   115     @{command_def "print_antiquotations"}\<open>\<^sup>*\<close> & : & \<open>context \<rightarrow>\<close> \\
   116     @{command_def "print_antiquotations"}\<open>\<^sup>*\<close> & : & \<open>context \<rightarrow>\<close> \\
   196       @@{antiquotation ML_structure} options @{syntax text} |
   197       @@{antiquotation ML_structure} options @{syntax text} |
   197       @@{antiquotation ML_functor} options @{syntax text} |
   198       @@{antiquotation ML_functor} options @{syntax text} |
   198       @@{antiquotation emph} options @{syntax text} |
   199       @@{antiquotation emph} options @{syntax text} |
   199       @@{antiquotation bold} options @{syntax text} |
   200       @@{antiquotation bold} options @{syntax text} |
   200       @@{antiquotation verbatim} options @{syntax text} |
   201       @@{antiquotation verbatim} options @{syntax text} |
       
   202       @@{antiquotation system_option} options @{syntax embedded} |
   201       @@{antiquotation session} options @{syntax embedded} |
   203       @@{antiquotation session} options @{syntax embedded} |
   202       @@{antiquotation path} options @{syntax embedded} |
   204       @@{antiquotation path} options @{syntax embedded} |
   203       @@{antiquotation "file"} options @{syntax name} |
   205       @@{antiquotation "file"} options @{syntax name} |
   204       @@{antiquotation dir} options @{syntax name} |
   206       @@{antiquotation dir} options @{syntax name} |
   205       @@{antiquotation url} options @{syntax embedded} |
   207       @@{antiquotation url} options @{syntax embedded} |
   287   \<^descr> \<open>@{bold s}\<close> prints document source recursively, with {\LaTeX} markup
   289   \<^descr> \<open>@{bold s}\<close> prints document source recursively, with {\LaTeX} markup
   288   \<^verbatim>\<open>\textbf{\<close>\<open>\<dots>\<close>\<^verbatim>\<open>}\<close>.
   290   \<^verbatim>\<open>\textbf{\<close>\<open>\<dots>\<close>\<^verbatim>\<open>}\<close>.
   289 
   291 
   290   \<^descr> \<open>@{verbatim s}\<close> prints uninterpreted source text literally as ASCII
   292   \<^descr> \<open>@{verbatim s}\<close> prints uninterpreted source text literally as ASCII
   291   characters, using some type-writer font style.
   293   characters, using some type-writer font style.
       
   294 
       
   295   \<^descr> \<open>@{system_option name}\<close> prints the given system option verbatim. The name
       
   296   is checked wrt.\ cumulative \<^verbatim>\<open>etc/options\<close> of all Isabelle components,
       
   297   notably \<^file>\<open>~~/etc/options\<close>.
   292 
   298 
   293   \<^descr> \<open>@{session name}\<close> prints given session name verbatim. The name is checked
   299   \<^descr> \<open>@{session name}\<close> prints given session name verbatim. The name is checked
   294   wrt.\ the dependencies of the current session.
   300   wrt.\ the dependencies of the current session.
   295 
   301 
   296   \<^descr> \<open>@{path name}\<close> prints the file-system path name verbatim.
   302   \<^descr> \<open>@{path name}\<close> prints the file-system path name verbatim.