src/Doc/System/Misc.thy
changeset 72309 564012e31db1
parent 71579 9b49538845cc
child 72316 3cc6aa405858
equal deleted inserted replaced
72308:aa14f630d8ef 72309:564012e31db1
   161   any sense for regular Isabelle releases. If the file already exists, it
   161   any sense for regular Isabelle releases. If the file already exists, it
   162   needs to be edited manually according to the printed explanation.
   162   needs to be edited manually according to the printed explanation.
   163 \<close>
   163 \<close>
   164 
   164 
   165 
   165 
   166 section \<open>Displaying documents \label{sec:tool-display}\<close>
       
   167 
       
   168 text \<open>
       
   169   The @{tool_def display} tool displays documents in DVI or PDF format:
       
   170   @{verbatim [display]
       
   171 \<open>Usage: isabelle display DOCUMENT
       
   172 
       
   173   Display DOCUMENT (in DVI or PDF format).\<close>}
       
   174 
       
   175   \<^medskip>
       
   176   The settings @{setting DVI_VIEWER} and @{setting PDF_VIEWER} determine the
       
   177   programs for viewing the corresponding file formats. Normally this opens the
       
   178   document via the desktop environment, potentially in an asynchronous manner
       
   179   with re-use of previews views.
       
   180 \<close>
       
   181 
       
   182 
       
   183 section \<open>Viewing documentation \label{sec:tool-doc}\<close>
   166 section \<open>Viewing documentation \label{sec:tool-doc}\<close>
   184 
   167 
   185 text \<open>
   168 text \<open>
   186   The @{tool_def doc} tool displays Isabelle documentation:
   169   The @{tool_def doc} tool displays Isabelle documentation:
   187   @{verbatim [display]
   170   @{verbatim [display]
   190   View Isabelle documentation.\<close>}
   173   View Isabelle documentation.\<close>}
   191 
   174 
   192   If called without arguments, it lists all available documents. Each line
   175   If called without arguments, it lists all available documents. Each line
   193   starts with an identifier, followed by a short description. Any of these
   176   starts with an identifier, followed by a short description. Any of these
   194   identifiers may be specified as arguments, in order to display the
   177   identifiers may be specified as arguments, in order to display the
   195   corresponding document (see also \secref{sec:tool-display}).
   178   corresponding document.
   196 
   179 
   197   \<^medskip>
   180   \<^medskip>
   198   The @{setting ISABELLE_DOCS} setting specifies the list of directories
   181   The @{setting ISABELLE_DOCS} setting specifies the list of directories
   199   (separated by colons) to be scanned for documentations.
   182   (separated by colons) to be scanned for documentations.
   200 \<close>
   183 \<close>