src/Doc/System/Sessions.thy
changeset 72574 d892f6d66402
parent 72515 c7038c397ae3
child 72600 2fa4f25d9d07
equal deleted inserted replaced
72573:a085a1a89388 72574:d892f6d66402
   188   in particular with document preparation (\chref{ch:present}).
   188   in particular with document preparation (\chref{ch:present}).
   189 
   189 
   190     \<^item> @{system_option_def "browser_info"} controls output of HTML browser
   190     \<^item> @{system_option_def "browser_info"} controls output of HTML browser
   191     info, see also \secref{sec:info}.
   191     info, see also \secref{sec:info}.
   192 
   192 
   193     \<^item> @{system_option_def "document"} specifies the document output format,
   193     \<^item> @{system_option_def "document"} controls document output for a
   194     see @{tool document} option \<^verbatim>\<open>-o\<close> in \secref{sec:tool-document}. In
   194     particular session or theory; \<^verbatim>\<open>document=pdf\<close> means enabled,
   195     practice, the most relevant values are \<^verbatim>\<open>document=false\<close> or
   195     \<^verbatim>\<open>document=false\<close> means disabled (especially for particular theories).
   196     \<^verbatim>\<open>document=pdf\<close>.
       
   197 
   196 
   198     \<^item> @{system_option_def "document_output"} specifies an alternative
   197     \<^item> @{system_option_def "document_output"} specifies an alternative
   199     directory for generated output of the document preparation system; the
   198     directory for generated output of the document preparation system; the
   200     default is within the @{setting "ISABELLE_BROWSER_INFO"} hierarchy as
   199     default is within the @{setting "ISABELLE_BROWSER_INFO"} hierarchy as
   201     explained in \secref{sec:info}. See also @{tool mkroot}, which generates a
   200     explained in \secref{sec:info}. See also @{tool mkroot}, which generates a
   202     default configuration with output readily available to the author of the
   201     default configuration with output readily available to the author of the
   203     document.
   202     document.
   204 
   203 
   205     \<^item> @{system_option_def "document_variants"} specifies document variants as
   204     \<^item> @{system_option_def "document_variants"} specifies document variants as
   206     a colon-separated list of \<open>name=tags\<close> entries, corresponding to @{tool
   205     a colon-separated list of \<open>name=tags\<close> entries. The default name
   207     document} options \<^verbatim>\<open>-n\<close> and \<^verbatim>\<open>-t\<close>.
   206     \<^verbatim>\<open>document\<close>, without additional tags.
   208 
   207 
   209     For example, \<^verbatim>\<open>document_variants=document:outline=/proof,/ML\<close> indicates
   208     Tags are specified as a comma separated list of modifier/name pairs and
       
   209     tell {\LaTeX} how to interpret certain Isabelle command regions:
       
   210     ``\<^verbatim>\<open>+\<close>\<open>foo\<close>'' (or just ``\<open>foo\<close>'') means to keep, ``\<^verbatim>\<open>-\<close>\<open>foo\<close>'' to drop,
       
   211     and ``\<^verbatim>\<open>/\<close>\<open>foo\<close>'' to fold text tagged as \<open>foo\<close>. The builtin default is
       
   212     equivalent to the tag specification
       
   213     ``\<^verbatim>\<open>+document,+theory,+proof,+ML,+visible,-invisible,+important,+unimportant\<close>'';
       
   214     see also the {\LaTeX} macros \<^verbatim>\<open>\isakeeptag\<close>, \<^verbatim>\<open>\isadroptag\<close>, and
       
   215     \<^verbatim>\<open>\isafoldtag\<close>, in \<^file>\<open>~~/lib/texinputs/isabelle.sty\<close>.
       
   216 
       
   217     In contrast, \<^verbatim>\<open>document_variants=document:outline=/proof,/ML\<close> indicates
   210     two documents: the one called \<^verbatim>\<open>document\<close> with default tags, and the other
   218     two documents: the one called \<^verbatim>\<open>document\<close> with default tags, and the other
   211     called \<^verbatim>\<open>outline\<close> where proofs and ML sections are folded.
   219     called \<^verbatim>\<open>outline\<close> where proofs and ML sections are folded.
   212 
   220 
   213     Document variant names are just a matter of conventions. It is also
   221     Document variant names are just a matter of conventions. It is also
   214     possible to use different document variant names (without tags) for
   222     possible to use different document variant names (without tags) for