src/Doc/System/Interfaces.thy
changeset 54703 499f92dc6e45
parent 54682 6587c627a9db
child 54881 dff57132cf18
equal deleted inserted replaced
54702:3daeba5130f0 54703:499f92dc6e45
     5 chapter {* User interfaces *}
     5 chapter {* User interfaces *}
     6 
     6 
     7 section {* Isabelle/jEdit Prover IDE \label{sec:tool-jedit} *}
     7 section {* Isabelle/jEdit Prover IDE \label{sec:tool-jedit} *}
     8 
     8 
     9 text {* The @{tool_def jedit} tool invokes a version of
     9 text {* The @{tool_def jedit} tool invokes a version of
    10   jEdit\footnote{\url{http://www.jedit.org/}} that has been augmented
    10   jEdit\footnote{@{url "http://www.jedit.org/"}} that has been augmented
    11   with some plugins to provide a fully-featured Prover IDE:
    11   with some plugins to provide a fully-featured Prover IDE:
    12 \begin{ttbox} Usage: isabelle jedit [OPTIONS]
    12 \begin{ttbox} Usage: isabelle jedit [OPTIONS]
    13   [FILES ...]
    13   [FILES ...]
    14 
    14 
    15   Options are:
    15   Options are:
    47 
    47 
    48   The @{verbatim "-b"} and @{verbatim "-f"} options control the
    48   The @{verbatim "-b"} and @{verbatim "-f"} options control the
    49   self-build mechanism of Isabelle/jEdit.  This is only relevant for
    49   self-build mechanism of Isabelle/jEdit.  This is only relevant for
    50   building from sources, which also requires an auxiliary @{verbatim
    50   building from sources, which also requires an auxiliary @{verbatim
    51   jedit_build}
    51   jedit_build}
    52   component.\footnote{\url{http://isabelle.in.tum.de/components}} Note
    52   component.\footnote{@{url "http://isabelle.in.tum.de/components"}} Note
    53   that official Isabelle releases already include a version of
    53   that official Isabelle releases already include a version of
    54   Isabelle/jEdit that is built properly.
    54   Isabelle/jEdit that is built properly.
    55 *}
    55 *}
    56 
    56 
    57 
    57 
    58 section {* Proof General / Emacs *}
    58 section {* Proof General / Emacs *}
    59 
    59 
    60 text {* The @{tool_def emacs} tool invokes a version of Emacs and
    60 text {* The @{tool_def emacs} tool invokes a version of Emacs and
    61   Proof General\footnote{http://proofgeneral.inf.ed.ac.uk/} within the
    61   Proof General\footnote{@{url "http://proofgeneral.inf.ed.ac.uk/"}} within the
    62   regular Isabelle settings environment (\secref{sec:settings}).  This
    62   regular Isabelle settings environment (\secref{sec:settings}).  This
    63   is more convenient than starting Emacs separately, loading the Proof
    63   is more convenient than starting Emacs separately, loading the Proof
    64   General LISP files, and then attempting to start Isabelle with
    64   General LISP files, and then attempting to start Isabelle with
    65   dynamic @{setting PATH} lookup etc., although it might fail if a
    65   dynamic @{setting PATH} lookup etc., although it might fail if a
    66   different version of Proof General is already part of the Emacs
    66   different version of Proof General is already part of the Emacs