src/Doc/System/Presentation.thy
changeset 61493 0debd22f0c0e
parent 61477 e467ae7aa808
child 61503 28e788ca2c5d
equal deleted inserted replaced
61492:3480725c71d2 61493:0debd22f0c0e
   113     -d           enable document preparation
   113     -d           enable document preparation
   114     -n NAME      alternative session name (default: DIR base name)
   114     -n NAME      alternative session name (default: DIR base name)
   115 
   115 
   116   Prepare session root DIR (default: current directory).\<close>}
   116   Prepare session root DIR (default: current directory).\<close>}
   117 
   117 
   118   The results are placed in the given directory @{text dir}, which
   118   The results are placed in the given directory \<open>dir\<close>, which
   119   refers to the current directory by default.  The @{tool mkroot} tool
   119   refers to the current directory by default.  The @{tool mkroot} tool
   120   is conservative in the sense that it does not overwrite existing
   120   is conservative in the sense that it does not overwrite existing
   121   files or directories.  Earlier attempts to generate a session root
   121   files or directories.  Earlier attempts to generate a session root
   122   need to be deleted manually.
   122   need to be deleted manually.
   123 
   123 
   124   \<^medskip>
   124   \<^medskip>
   125   Option @{verbatim "-d"} indicates that the session shall be
   125   Option @{verbatim "-d"} indicates that the session shall be
   126   accompanied by a formal document, with @{text DIR}@{verbatim
   126   accompanied by a formal document, with \<open>DIR\<close>@{verbatim
   127   "/document/root.tex"} as its {\LaTeX} entry point (see also
   127   "/document/root.tex"} as its {\LaTeX} entry point (see also
   128   \chref{ch:present}).
   128   \chref{ch:present}).
   129 
   129 
   130   Option @{verbatim "-n"} allows to specify an alternative session
   130   Option @{verbatim "-n"} allows to specify an alternative session
   131   name; otherwise the base name of the given directory is used.
   131   name; otherwise the base name of the given directory is used.
   186   the target @{verbatim DIR}.
   186   the target @{verbatim DIR}.
   187 
   187 
   188   \<^medskip>
   188   \<^medskip>
   189   The @{verbatim "-t"} option tells {\LaTeX} how to interpret
   189   The @{verbatim "-t"} option tells {\LaTeX} how to interpret
   190   tagged Isabelle command regions.  Tags are specified as a comma
   190   tagged Isabelle command regions.  Tags are specified as a comma
   191   separated list of modifier/name pairs: ``@{verbatim "+"}@{text
   191   separated list of modifier/name pairs: ``@{verbatim "+"}\<open>foo\<close>'' (or just ``\<open>foo\<close>'') means to keep, ``@{verbatim
   192   foo}'' (or just ``@{text foo}'') means to keep, ``@{verbatim
   192   "-"}\<open>foo\<close>'' to drop, and ``@{verbatim "/"}\<open>foo\<close>'' to
   193   "-"}@{text foo}'' to drop, and ``@{verbatim "/"}@{text foo}'' to
   193   fold text tagged as \<open>foo\<close>.  The builtin default is equivalent
   194   fold text tagged as @{text foo}.  The builtin default is equivalent
       
   195   to the tag specification ``@{verbatim
   194   to the tag specification ``@{verbatim
   196   "+theory,+proof,+ML,+visible,-invisible"}''; see also the {\LaTeX}
   195   "+theory,+proof,+ML,+visible,-invisible"}''; see also the {\LaTeX}
   197   macros @{verbatim "\\isakeeptag"}, @{verbatim "\\isadroptag"}, and
   196   macros @{verbatim "\\isakeeptag"}, @{verbatim "\\isadroptag"}, and
   198   @{verbatim "\\isafoldtag"}, in @{file
   197   @{verbatim "\\isafoldtag"}, in @{file
   199   "~~/lib/texinputs/isabelle.sty"}.
   198   "~~/lib/texinputs/isabelle.sty"}.
   223 
   222 
   224   \<^medskip>
   223   \<^medskip>
   225   When running the session, Isabelle copies the content of
   224   When running the session, Isabelle copies the content of
   226   the original @{verbatim document} directory into its proper place
   225   the original @{verbatim document} directory into its proper place
   227   within @{setting ISABELLE_BROWSER_INFO}, according to the session
   226   within @{setting ISABELLE_BROWSER_INFO}, according to the session
   228   path and document variant.  Then, for any processed theory @{text A}
   227   path and document variant.  Then, for any processed theory \<open>A\<close>
   229   some {\LaTeX} source is generated and put there as @{text
   228   some {\LaTeX} source is generated and put there as \<open>A\<close>@{verbatim ".tex"}.  Furthermore, a list of all generated theory
   230   A}@{verbatim ".tex"}.  Furthermore, a list of all generated theory
       
   231   files is put into @{verbatim session.tex}.  Typically, the root
   229   files is put into @{verbatim session.tex}.  Typically, the root
   232   {\LaTeX} file provided by the user would include @{verbatim
   230   {\LaTeX} file provided by the user would include @{verbatim
   233   session.tex} to get a document containing all the theories.
   231   session.tex} to get a document containing all the theories.
   234 
   232 
   235   The {\LaTeX} versions of the theories require some macros defined in
   233   The {\LaTeX} versions of the theories require some macros defined in
   240 
   238 
   241   If the text contains any references to Isabelle symbols (such as
   239   If the text contains any references to Isabelle symbols (such as
   242   @{verbatim "\\"}@{verbatim "<forall>"}) then @{verbatim
   240   @{verbatim "\\"}@{verbatim "<forall>"}) then @{verbatim
   243   "isabellesym.sty"} should be included as well.  This package
   241   "isabellesym.sty"} should be included as well.  This package
   244   contains a standard set of {\LaTeX} macro definitions @{verbatim
   242   contains a standard set of {\LaTeX} macro definitions @{verbatim
   245   "\\isasym"}@{text foo} corresponding to @{verbatim "\\"}@{verbatim
   243   "\\isasym"}\<open>foo\<close> corresponding to @{verbatim "\\"}@{verbatim
   246   "<"}@{text foo}@{verbatim ">"}, see @{cite "isabelle-implementation"} for a
   244   "<"}\<open>foo\<close>@{verbatim ">"}, see @{cite "isabelle-implementation"} for a
   247   complete list of predefined Isabelle symbols.  Users may invent
   245   complete list of predefined Isabelle symbols.  Users may invent
   248   further symbols as well, just by providing {\LaTeX} macros in a
   246   further symbols as well, just by providing {\LaTeX} macros in a
   249   similar fashion as in @{file "~~/lib/texinputs/isabellesym.sty"} of
   247   similar fashion as in @{file "~~/lib/texinputs/isabellesym.sty"} of
   250   the Isabelle distribution.
   248   the Isabelle distribution.
   251 
   249