src/Doc/System/Presentation.thy
changeset 72309 564012e31db1
parent 67399 eab6ce8368fa
child 72574 d892f6d66402
equal deleted inserted replaced
72308:aa14f630d8ef 72309:564012e31db1
   151 \<open>Usage: isabelle document [OPTIONS]
   151 \<open>Usage: isabelle document [OPTIONS]
   152 
   152 
   153   Options are:
   153   Options are:
   154     -d DIR       document output directory (default "output/document")
   154     -d DIR       document output directory (default "output/document")
   155     -n NAME      document name (default "document")
   155     -n NAME      document name (default "document")
   156     -o FORMAT    document format: pdf (default), dvi
       
   157     -t TAGS      markup for tagged regions
   156     -t TAGS      markup for tagged regions
   158 
   157 
   159   Prepare the theory session document in document directory, producing the
   158   Prepare the theory session document in document directory, producing the
   160   specified output format.
   159   specified output format.
   161 \<close>}
   160 \<close>}
   170   Option \<^verbatim>\<open>-d\<close> specifies an alternative document output directory. The default
   169   Option \<^verbatim>\<open>-d\<close> specifies an alternative document output directory. The default
   171   is \<^verbatim>\<open>output/document\<close> (derived from the document name). Note that the result
   170   is \<^verbatim>\<open>output/document\<close> (derived from the document name). Note that the result
   172   will appear in the parent of this directory.
   171   will appear in the parent of this directory.
   173 
   172 
   174   \<^medskip>
   173   \<^medskip>
   175   The \<^verbatim>\<open>-n\<close> and \<^verbatim>\<open>-o\<close> option specify the final output file name and format,
   174   Option \<^verbatim>\<open>-n\<close> specifies the resulting document file name, the default is
   176   the default is ``\<^verbatim>\<open>document.pdf\<close>''.
   175   ``\<^verbatim>\<open>document\<close>'' (leading to ``\<^verbatim>\<open>document.pdf\<close>'').
   177 
   176 
   178   \<^medskip>
   177   \<^medskip>
   179   The \<^verbatim>\<open>-t\<close> option tells {\LaTeX} how to interpret tagged Isabelle command
   178   The \<^verbatim>\<open>-t\<close> option tells {\LaTeX} how to interpret tagged Isabelle command
   180   regions. Tags are specified as a comma separated list of modifier/name
   179   regions. Tags are specified as a comma separated list of modifier/name
   181   pairs: ``\<^verbatim>\<open>+\<close>\<open>foo\<close>'' (or just ``\<open>foo\<close>'') means to keep, ``\<^verbatim>\<open>-\<close>\<open>foo\<close>'' to
   180   pairs: ``\<^verbatim>\<open>+\<close>\<open>foo\<close>'' (or just ``\<open>foo\<close>'') means to keep, ``\<^verbatim>\<open>-\<close>\<open>foo\<close>'' to
   227   \<^verbatim>\<open>\\<close>\<^verbatim>\<open><\<close>\<open>foo\<close>\<^verbatim>\<open>>\<close>, see @{cite "isabelle-implementation"} for a complete list
   226   \<^verbatim>\<open>\\<close>\<^verbatim>\<open><\<close>\<open>foo\<close>\<^verbatim>\<open>>\<close>, see @{cite "isabelle-implementation"} for a complete list
   228   of predefined Isabelle symbols. Users may invent further symbols as well,
   227   of predefined Isabelle symbols. Users may invent further symbols as well,
   229   just by providing {\LaTeX} macros in a similar fashion as in
   228   just by providing {\LaTeX} macros in a similar fashion as in
   230   \<^file>\<open>~~/lib/texinputs/isabellesym.sty\<close> of the Isabelle distribution.
   229   \<^file>\<open>~~/lib/texinputs/isabellesym.sty\<close> of the Isabelle distribution.
   231 
   230 
   232   For proper setup of DVI and PDF documents (with hyperlinks and bookmarks),
   231   For proper setup of PDF documents (with hyperlinks and bookmarks),
   233   we recommend to include \<^file>\<open>~~/lib/texinputs/pdfsetup.sty\<close> as well.
   232   we recommend to include \<^file>\<open>~~/lib/texinputs/pdfsetup.sty\<close> as well.
   234 
   233 
   235   \<^medskip>
   234   \<^medskip>
   236   As a final step of Isabelle document preparation, @{tool document} is run on
   235   As a final step of Isabelle document preparation, @{tool document} is run on
   237   the generated \<^verbatim>\<open>output/document\<close> directory. Thus the actual output document
   236   the generated \<^verbatim>\<open>output/document\<close> directory. Thus the actual output document
   252   document preparation. Its usage is:
   251   document preparation. Its usage is:
   253   @{verbatim [display]
   252   @{verbatim [display]
   254 \<open>Usage: isabelle latex [OPTIONS] [FILE]
   253 \<open>Usage: isabelle latex [OPTIONS] [FILE]
   255 
   254 
   256   Options are:
   255   Options are:
   257     -o FORMAT    specify output format: pdf (default), dvi, bbl, idx, sty
   256     -o FORMAT    specify output format: pdf (default), bbl, idx, sty
   258 
   257 
   259   Run LaTeX (and related tools) on FILE (default root.tex),
   258   Run LaTeX (and related tools) on FILE (default root.tex),
   260   producing the specified output format.\<close>}
   259   producing the specified output format.\<close>}
   261 
   260 
   262   Appropriate {\LaTeX}-related programs are run on the input file, according
   261   Appropriate {\LaTeX}-related programs are run on the input file, according
   263   to the given output format: @{executable latex}, @{executable pdflatex},
   262   to the given output format: @{executable pdflatex}, @{executable bibtex}
   264   @{executable dvips}, @{executable bibtex} (for \<^verbatim>\<open>bbl\<close>), and @{executable
   263   (for \<^verbatim>\<open>bbl\<close>), and @{executable makeindex} (for \<^verbatim>\<open>idx\<close>). The actual commands
   265   makeindex} (for \<^verbatim>\<open>idx\<close>). The actual commands are determined from the
   264   are determined from the settings environment (@{setting ISABELLE_PDFLATEX}
   266   settings environment (@{setting ISABELLE_PDFLATEX} etc.).
   265   etc.).
   267 
   266 
   268   The \<^verbatim>\<open>sty\<close> output format causes the Isabelle style files to be updated from
   267   The \<^verbatim>\<open>sty\<close> output format causes the Isabelle style files to be updated from
   269   the distribution. This is useful in special situations where the document
   268   the distribution. This is useful in special situations where the document
   270   sources are to be processed another time by separate tools.
   269   sources are to be processed another time by separate tools.
   271 \<close>
   270 \<close>