src/Doc/System/Misc.thy
changeset 57443 577f029fde39
parent 57439 0e41f26a0250
child 58618 782f0b662cae
equal deleted inserted replaced
57442:2373b4c61111 57443:577f029fde39
   307   \medskip The @{setting ISABELLE_DOCS} setting specifies the list of
   307   \medskip The @{setting ISABELLE_DOCS} setting specifies the list of
   308   directories (separated by colons) to be scanned for documentations.
   308   directories (separated by colons) to be scanned for documentations.
   309 *}
   309 *}
   310 
   310 
   311 
   311 
   312 section {* Proof General / Emacs *}
       
   313 
       
   314 text {* The @{tool_def emacs} tool invokes a version of Emacs and
       
   315   Proof General\footnote{@{url "http://proofgeneral.inf.ed.ac.uk/"}} within the
       
   316   regular Isabelle settings environment (\secref{sec:settings}).  This
       
   317   is more convenient than starting Emacs separately, loading the Proof
       
   318   General LISP files, and then attempting to start Isabelle with
       
   319   dynamic @{setting PATH} lookup etc., although it might fail if a
       
   320   different version of Proof General is already part of the Emacs
       
   321   installation of the operating system.
       
   322 
       
   323   The actual interface script is part of the Proof General
       
   324   distribution; its usage depends on the particular version.  There
       
   325   are some options available, such as @{verbatim "-l"} for passing the
       
   326   logic image to be used by default, or @{verbatim "-m"} to tune the
       
   327   standard print mode of the prover process.  The following Isabelle
       
   328   settings are particularly important for Proof General:
       
   329 
       
   330   \begin{description}
       
   331 
       
   332   \item[@{setting_def PROOFGENERAL_HOME}] points to the main
       
   333   installation directory of the Proof General distribution.  This is
       
   334   implicitly provided for versions of Proof General that are
       
   335   distributed as Isabelle component, see also \secref{sec:components};
       
   336   otherwise it needs to be configured manually.
       
   337 
       
   338   \item[@{setting_def PROOFGENERAL_OPTIONS}] is implicitly prefixed to
       
   339   the command line of any invocation of the Proof General @{verbatim
       
   340   interface} script.  This allows to provide persistent default
       
   341   options for the invocation of \texttt{isabelle emacs}.
       
   342 
       
   343   \end{description}
       
   344 *}
       
   345 
       
   346 
       
   347 section {* Shell commands within the settings environment \label{sec:tool-env} *}
   312 section {* Shell commands within the settings environment \label{sec:tool-env} *}
   348 
   313 
   349 text {* The @{tool_def env} tool is a direct wrapper for the standard
   314 text {* The @{tool_def env} tool is a direct wrapper for the standard
   350   @{verbatim "/usr/bin/env"} command on POSIX systems, running within
   315   @{verbatim "/usr/bin/env"} command on POSIX systems, running within
   351   the Isabelle settings environment (\secref{sec:settings}).
   316   the Isabelle settings environment (\secref{sec:settings}).