src/Doc/System/Presentation.thy
changeset 72309 564012e31db1
parent 67399 eab6ce8368fa
child 72574 d892f6d66402
--- a/src/Doc/System/Presentation.thy	Sat Sep 26 11:43:25 2020 +0200
+++ b/src/Doc/System/Presentation.thy	Sat Sep 26 14:29:46 2020 +0200
@@ -153,7 +153,6 @@
   Options are:
     -d DIR       document output directory (default "output/document")
     -n NAME      document name (default "document")
-    -o FORMAT    document format: pdf (default), dvi
     -t TAGS      markup for tagged regions
 
   Prepare the theory session document in document directory, producing the
@@ -172,8 +171,8 @@
   will appear in the parent of this directory.
 
   \<^medskip>
-  The \<^verbatim>\<open>-n\<close> and \<^verbatim>\<open>-o\<close> option specify the final output file name and format,
-  the default is ``\<^verbatim>\<open>document.pdf\<close>''.
+  Option \<^verbatim>\<open>-n\<close> specifies the resulting document file name, the default is
+  ``\<^verbatim>\<open>document\<close>'' (leading to ``\<^verbatim>\<open>document.pdf\<close>'').
 
   \<^medskip>
   The \<^verbatim>\<open>-t\<close> option tells {\LaTeX} how to interpret tagged Isabelle command
@@ -229,7 +228,7 @@
   just by providing {\LaTeX} macros in a similar fashion as in
   \<^file>\<open>~~/lib/texinputs/isabellesym.sty\<close> of the Isabelle distribution.
 
-  For proper setup of DVI and PDF documents (with hyperlinks and bookmarks),
+  For proper setup of PDF documents (with hyperlinks and bookmarks),
   we recommend to include \<^file>\<open>~~/lib/texinputs/pdfsetup.sty\<close> as well.
 
   \<^medskip>
@@ -254,16 +253,16 @@
 \<open>Usage: isabelle latex [OPTIONS] [FILE]
 
   Options are:
-    -o FORMAT    specify output format: pdf (default), dvi, bbl, idx, sty
+    -o FORMAT    specify output format: pdf (default), bbl, idx, sty
 
   Run LaTeX (and related tools) on FILE (default root.tex),
   producing the specified output format.\<close>}
 
   Appropriate {\LaTeX}-related programs are run on the input file, according
-  to the given output format: @{executable latex}, @{executable pdflatex},
-  @{executable dvips}, @{executable bibtex} (for \<^verbatim>\<open>bbl\<close>), and @{executable
-  makeindex} (for \<^verbatim>\<open>idx\<close>). The actual commands are determined from the
-  settings environment (@{setting ISABELLE_PDFLATEX} etc.).
+  to the given output format: @{executable pdflatex}, @{executable bibtex}
+  (for \<^verbatim>\<open>bbl\<close>), and @{executable makeindex} (for \<^verbatim>\<open>idx\<close>). The actual commands
+  are determined from the settings environment (@{setting ISABELLE_PDFLATEX}
+  etc.).
 
   The \<^verbatim>\<open>sty\<close> output format causes the Isabelle style files to be updated from
   the distribution. This is useful in special situations where the document