doc-src/System/Thy/Presentation.thy
changeset 28914 f993cbffc42a
parent 28838 d5db6dfcb34a
child 29435 a5f84ac14609
equal deleted inserted replaced
28913:86ed1c86e0ef 28914:f993cbffc42a
    91 
    91 
    92   and then change into the @{"file" "~~/src/FOL"} directory and run
    92   and then change into the @{"file" "~~/src/FOL"} directory and run
    93   @{verbatim isabelle} @{tool make}, or even @{verbatim isabelle} @{tool
    93   @{verbatim isabelle} @{tool make}, or even @{verbatim isabelle} @{tool
    94   make}~@{verbatim all}.  The presentation output will appear in
    94   make}~@{verbatim all}.  The presentation output will appear in
    95   @{verbatim "ISABELLE_BROWSER_INFO/FOL"}, which usually refers to
    95   @{verbatim "ISABELLE_BROWSER_INFO/FOL"}, which usually refers to
    96   @{verbatim "~/isabelle/browser_info/FOL"}.  Note that option
    96   @{verbatim "~/.isabelle/browser_info/FOL"}.  Note that option
    97   @{verbatim "-v true"} will make the internal runs of @{tool usedir}
    97   @{verbatim "-v true"} will make the internal runs of @{tool usedir}
    98   more explicit about such details.
    98   more explicit about such details.
    99 
    99 
   100   Many standard Isabelle sessions (such as @{"file" "~~/src/HOL/ex"})
   100   Many standard Isabelle sessions (such as @{"file" "~~/src/HOL/ex"})
   101   also provide actual printable documents.  These are prepared
   101   also provide actual printable documents.  These are prepared
   754   process leaves the sources at a certain place within @{setting
   754   process leaves the sources at a certain place within @{setting
   755   ISABELLE_BROWSER_INFO}, see the runtime error message for details.
   755   ISABELLE_BROWSER_INFO}, see the runtime error message for details.
   756   This enables users to inspect {\LaTeX} runs in further detail, e.g.\
   756   This enables users to inspect {\LaTeX} runs in further detail, e.g.\
   757   like this:
   757   like this:
   758 \begin{ttbox}
   758 \begin{ttbox}
   759   cd ~/isabelle/browser_info/HOL/Test/document
   759   cd ~/.isabelle/browser_info/HOL/Test/document
   760   isabelle latex -o pdf
   760   isabelle latex -o pdf
   761 \end{ttbox}
   761 \end{ttbox}
   762 *}
   762 *}
   763 
   763 
   764 end
   764 end