src/Doc/System/Sessions.thy
changeset 74873 0ab2ed1489eb
parent 74827 c1b5d6e6ff74
child 75161 95612f330c93
equal deleted inserted replaced
74872:9e9a308562da 74873:0ab2ed1489eb
   210     default is within the @{setting "ISABELLE_BROWSER_INFO"} hierarchy as
   210     default is within the @{setting "ISABELLE_BROWSER_INFO"} hierarchy as
   211     explained in \secref{sec:info}. See also @{tool mkroot}, which generates a
   211     explained in \secref{sec:info}. See also @{tool mkroot}, which generates a
   212     default configuration with output readily available to the author of the
   212     default configuration with output readily available to the author of the
   213     document.
   213     document.
   214 
   214 
       
   215     \<^item> @{system_option_def "document_echo"} informs about document file names
       
   216     during session presentation.
       
   217 
   215     \<^item> @{system_option_def "document_variants"} specifies document variants as
   218     \<^item> @{system_option_def "document_variants"} specifies document variants as
   216     a colon-separated list of \<open>name=tags\<close> entries. The default name
   219     a colon-separated list of \<open>name=tags\<close> entries. The default name
   217     \<^verbatim>\<open>document\<close>, without additional tags.
   220     \<^verbatim>\<open>document\<close>, without additional tags.
   218 
   221 
   219     Tags are specified as a comma separated list of modifier/name pairs and
   222     Tags are specified as a comma separated list of modifier/name pairs and
   237     as a comma-separated list of items: either ``\<open>command\<close>\<^verbatim>\<open>%\<close>\<open>tag\<close>'' for a
   240     as a comma-separated list of items: either ``\<open>command\<close>\<^verbatim>\<open>%\<close>\<open>tag\<close>'' for a
   238     specific command, or ``\<^verbatim>\<open>%\<close>\<open>tag\<close>'' as default for all other commands. This
   241     specific command, or ``\<^verbatim>\<open>%\<close>\<open>tag\<close>'' as default for all other commands. This
   239     is occasionally useful to control the global visibility of commands via
   242     is occasionally useful to control the global visibility of commands via
   240     session options (e.g.\ in \<^verbatim>\<open>ROOT\<close>).
   243     session options (e.g.\ in \<^verbatim>\<open>ROOT\<close>).
   241 
   244 
       
   245     \<^item> @{system_option_def "document_comment_latex"} enables regular {\LaTeX}
       
   246     \<^verbatim>\<open>comment.sty\<close>, instead of the historic version for plain {\TeX}
       
   247     (default). The latter is much faster, but in conflict with {\LaTeX}
       
   248     classes like Dagstuhl
       
   249     LIPIcs\<^footnote>\<open>\<^url>\<open>https://github.com/dagstuhl-publishing/styles\<close>\<close>.
       
   250 
   242     \<^item> @{system_option_def "document_bibliography"} explicitly enables the use
   251     \<^item> @{system_option_def "document_bibliography"} explicitly enables the use
   243     of \<^verbatim>\<open>bibtex\<close>; the default is to check the presence of \<^verbatim>\<open>root.bib\<close>, but it
   252     of \<^verbatim>\<open>bibtex\<close>; the default is to check the presence of \<^verbatim>\<open>root.bib\<close>, but it
   244     could have a different name.
   253     could have a different name.
       
   254 
       
   255     \<^item> @{system_option_def "document_heading_prefix"} specifies a prefix for
       
   256     the {\LaTeX} macro names generated from Isar commands like \<^theory_text>\<open>chapter\<close>,
       
   257     \<^theory_text>\<open>section\<close> etc. The default is \<^verbatim>\<open>isamarkup\<close>, e.g. \<^theory_text>\<open>section\<close> becomes
       
   258     \<^verbatim>\<open>\isamarkupsection\<close>.
   245 
   259 
   246     \<^item> @{system_option_def "threads"} determines the number of worker threads
   260     \<^item> @{system_option_def "threads"} determines the number of worker threads
   247     for parallel checking of theories and proofs. The default \<open>0\<close> means that a
   261     for parallel checking of theories and proofs. The default \<open>0\<close> means that a
   248     sensible maximum value is determined by the underlying hardware. For
   262     sensible maximum value is determined by the underlying hardware. For
   249     machines with many cores or with hyperthreading, this is often requires
   263     machines with many cores or with hyperthreading, this is often requires