doc-src/System/Thy/Misc.thy
changeset 28248 b2869ebcf8e3
parent 28238 398bf960d3d4
child 28253 04fc1ba19f93
equal deleted inserted replaced
28247:8aa636a9e2ce 28248:b2869ebcf8e3
     7 chapter {* Miscellaneous tools \label{ch:tools} *}
     7 chapter {* Miscellaneous tools \label{ch:tools} *}
     8 
     8 
     9 text {*
     9 text {*
    10   Subsequently we describe various Isabelle related utilities, given
    10   Subsequently we describe various Isabelle related utilities, given
    11   in alphabetical order.
    11   in alphabetical order.
       
    12 *}
       
    13 
       
    14 
       
    15 section {* The Proof General / Emacs interface *}
       
    16 
       
    17 text {*
       
    18   The @{tool_def emacs} tool invokes a version of Emacs with Proof
       
    19   General within the regular Isabelle settings environment
       
    20   (\secref{sec:settings}).  This is more robust than starting Emacs
       
    21   separately, loading the Proof General lisp files, and then
       
    22   attempting to start Isabelle with dynamic @{setting PATH} lookup
       
    23   etc.
       
    24 
       
    25   The actual interface script is part of the Proof General
       
    26   distribution~\cite{proofgeneral}; its usage depends on the
       
    27   particular version.  There are some options available, such as
       
    28   @{verbatim "-l"} for passing the logic image to be used by default,
       
    29   or @{verbatim "-m"} to tune the standard print mode.
       
    30 
       
    31   The following Isabelle settings are particularly important for Proof
       
    32   General:
       
    33 
       
    34   \begin{description}
       
    35 
       
    36   \item[@{setting_def PROOFGENERAL_HOME}] points to the main
       
    37   installation directory of the Proof General distribution.  The
       
    38   default settings try to locate this in a number of standard places,
       
    39   notably @{verbatim "$ISABELLE_HOME/contrib/ProofGeneral"}.
       
    40 
       
    41   \item[@{setting_def PROOFGENERAL_OPTIONS}] is implicitly prefixed to
       
    42   the command line of any invocation of the Proof General @{verbatim
       
    43   interface} script.
       
    44 
       
    45   \item[@{setting_def XSYMBOL_INSTALLFONTS}] may contain a small shell
       
    46   script to install the X11 fonts required for the X-Symbols mode of
       
    47   Proof General.  This is only required if the X11 display server runs
       
    48   on a different machine than the Emacs application, with a different
       
    49   file-system view on the Proof General installation.  Under most
       
    50   circumstances Proof General is able to refer to the font files that
       
    51   are part of its distribution.
       
    52 
       
    53   \end{description}
    12 *}
    54 *}
    13 
    55 
    14 
    56 
    15 section {* Displaying documents *}
    57 section {* Displaying documents *}
    16 
    58