src/Doc/Isar_Ref/Document_Preparation.thy
changeset 60270 a147272b16f9
parent 59937 6eccb133d4e6
child 60286 410115884a92
equal deleted inserted replaced
60269:652a8e72cb75 60270:a147272b16f9
     9   within that format.  This allows to produce papers, books, theses
     9   within that format.  This allows to produce papers, books, theses
    10   etc.\ from Isabelle theory sources.
    10   etc.\ from Isabelle theory sources.
    11 
    11 
    12   {\LaTeX} output is generated while processing a \emph{session} in
    12   {\LaTeX} output is generated while processing a \emph{session} in
    13   batch mode, as explained in the \emph{The Isabelle System Manual}
    13   batch mode, as explained in the \emph{The Isabelle System Manual}
    14   @{cite "isabelle-sys"}.  The main Isabelle tools to get started with
    14   @{cite "isabelle-system"}.  The main Isabelle tools to get started with
    15   document preparation are @{tool_ref mkroot} and @{tool_ref build}.
    15   document preparation are @{tool_ref mkroot} and @{tool_ref build}.
    16 
    16 
    17   The classic Isabelle/HOL tutorial @{cite "isabelle-hol-book"} also
    17   The classic Isabelle/HOL tutorial @{cite "isabelle-hol-book"} also
    18   explains some aspects of theory presentation.\<close>
    18   explains some aspects of theory presentation.\<close>
    19 
    19 
   432     @{text "proof"} & all proof commands \\
   432     @{text "proof"} & all proof commands \\
   433     @{text "ML"} & all commands involving ML code \\
   433     @{text "ML"} & all commands involving ML code \\
   434   \end{tabular}
   434   \end{tabular}
   435 
   435 
   436   \medskip The Isabelle document preparation system
   436   \medskip The Isabelle document preparation system
   437   @{cite "isabelle-sys"} allows tagged command regions to be presented
   437   @{cite "isabelle-system"} allows tagged command regions to be presented
   438   specifically, e.g.\ to fold proof texts, or drop parts of the text
   438   specifically, e.g.\ to fold proof texts, or drop parts of the text
   439   completely.
   439   completely.
   440 
   440 
   441   For example ``@{command "by"}~@{text "%invisible auto"}'' causes
   441   For example ``@{command "by"}~@{text "%invisible auto"}'' causes
   442   that piece of proof to be treated as @{text invisible} instead of
   442   that piece of proof to be treated as @{text invisible} instead of
   457   by the document author.  The Isabelle document preparation tools
   457   by the document author.  The Isabelle document preparation tools
   458   also provide some high-level options to specify the meaning of
   458   also provide some high-level options to specify the meaning of
   459   arbitrary tags to ``keep'', ``drop'', or ``fold'' the corresponding
   459   arbitrary tags to ``keep'', ``drop'', or ``fold'' the corresponding
   460   parts of the text.  Logic sessions may also specify ``document
   460   parts of the text.  Logic sessions may also specify ``document
   461   versions'', where given tags are interpreted in some particular way.
   461   versions'', where given tags are interpreted in some particular way.
   462   Again see @{cite "isabelle-sys"} for further details.
   462   Again see @{cite "isabelle-system"} for further details.
   463 \<close>
   463 \<close>
   464 
   464 
   465 
   465 
   466 section \<open>Railroad diagrams\<close>
   466 section \<open>Railroad diagrams\<close>
   467 
   467