src/Doc/System/Presentation.thy
changeset 72675 cc1347c8c804
parent 72653 ea35afdb1366
child 73724 5a3a2a52648d
equal deleted inserted replaced
72674:a9fea3f11cc0 72675:cc1347c8c804
   127   is:
   127   is:
   128   @{verbatim [display]
   128   @{verbatim [display]
   129 \<open>Usage: isabelle document [OPTIONS] SESSION
   129 \<open>Usage: isabelle document [OPTIONS] SESSION
   130 
   130 
   131   Options are:
   131   Options are:
   132     -O           set option "document_output", relative to current directory
   132     -O DIR       output directory for LaTeX sources and resulting PDF
       
   133     -P DIR       output directory for resulting PDF
       
   134     -S DIR       output directory for LaTeX sources
   133     -V           verbose latex
   135     -V           verbose latex
   134     -d DIR       include session directory
   136     -d DIR       include session directory
   135     -o OPTION    override Isabelle system OPTION (via NAME=VAL or NAME)
   137     -o OPTION    override Isabelle system OPTION (via NAME=VAL or NAME)
   136     -v           verbose build
   138     -v           verbose build
   137 
   139 
   146   \<^medskip> Options \<^verbatim>\<open>-d\<close>, \<^verbatim>\<open>-o\<close>, \<^verbatim>\<open>-v\<close> have the same meaning as for @{tool
   148   \<^medskip> Options \<^verbatim>\<open>-d\<close>, \<^verbatim>\<open>-o\<close>, \<^verbatim>\<open>-v\<close> have the same meaning as for @{tool
   147   build}.
   149   build}.
   148 
   150 
   149   \<^medskip> Option \<^verbatim>\<open>-V\<close> prints full output of {\LaTeX} tools.
   151   \<^medskip> Option \<^verbatim>\<open>-V\<close> prints full output of {\LaTeX} tools.
   150 
   152 
   151   \<^medskip> Option \<^verbatim>\<open>-O\<close>~\<open>dir\<close> specifies the @{system_option document_output} option
   153   \<^medskip> Option \<^verbatim>\<open>-O\<close>~\<open>dir\<close> specifies the output directory for generated {\LaTeX}
   152   relative to the current directory, while \<^verbatim>\<open>-o document_output=\<close>\<open>dir\<close> is
   154   sources and the result PDF file. Options \<^verbatim>\<open>-P\<close> and \<^verbatim>\<open>-S\<close> only refer to the
   153   relative to the session directory.
   155   PDF and sources, respectively.
   154 
   156 
   155   For example, for output directory ``\<^verbatim>\<open>output\<close>'' and the default document
   157   For example, for output directory ``\<^verbatim>\<open>output\<close>'' and the default document
   156   variant ``\<^verbatim>\<open>document\<close>'', the generated document sources are placed into the
   158   variant ``\<^verbatim>\<open>document\<close>'', the generated document sources are placed into the
   157   subdirectory \<^verbatim>\<open>output/document/\<close> and the resulting PDF into
   159   subdirectory \<^verbatim>\<open>output/document/\<close> and the resulting PDF into
   158   \<^verbatim>\<open>output/document.pdf\<close>.
   160   \<^verbatim>\<open>output/document.pdf\<close>.