doc-src/System/Thy/Basics.thy
changeset 28223 eee194395fdc
parent 28215 a1cfc43ac47d
child 28238 398bf960d3d4
equal deleted inserted replaced
28222:402a3f30542f 28223:eee194395fdc
    16   \medskip The Isabelle system environment emerges from a few general
    16   \medskip The Isabelle system environment emerges from a few general
    17   concepts.
    17   concepts.
    18 
    18 
    19   \begin{itemize}
    19   \begin{itemize}
    20 
    20 
    21   \item The \emph{Isabelle settings mechanism} provides environment variables to
    21   \item The \emph{Isabelle settings mechanism} provides environment
    22   all Isabelle programs (including tools and user interfaces).
    22   variables to all Isabelle programs (including tools and user
       
    23   interfaces).
    23 
    24 
    24   \item The \emph{Isabelle tools wrapper} (@{executable_def isatool})
    25   \item The \emph{Isabelle tools wrapper} (@{executable_def isatool})
    25   provides a generic startup platform for Isabelle related utilities.
    26   provides a generic startup platform for Isabelle related utilities.
    26   Thus tools automatically benefit from the settings mechanism.
    27   Thus tools automatically benefit from the settings mechanism.
    27 
    28 
   274 
   275 
   275 section {* The Isabelle tools wrapper \label{sec:isatool} *}
   276 section {* The Isabelle tools wrapper \label{sec:isatool} *}
   276 
   277 
   277 text {*
   278 text {*
   278   All Isabelle related utilities are called via a common wrapper ---
   279   All Isabelle related utilities are called via a common wrapper ---
   279   \ttindex{isatool}:
   280   @{executable isatool}:
   280 
   281 
   281 \begin{ttbox}
   282 \begin{ttbox}
   282 Usage: isatool TOOL [ARGS ...]
   283 Usage: isatool TOOL [ARGS ...]
   283 
   284 
   284   Start Isabelle utility program TOOL with ARGS. Pass "-?" to TOOL
   285   Start Isabelle utility program TOOL with ARGS. Pass "-?" to TOOL
   370   slash (@{verbatim "/"}) in the name (hint: use @{verbatim "./"} to
   371   slash (@{verbatim "/"}) in the name (hint: use @{verbatim "./"} to
   371   refer to the current directory).
   372   refer to the current directory).
   372 *}
   373 *}
   373 
   374 
   374 
   375 
   375 subsection {* Options *}
   376 subsubsection {* Options *}
   376 
   377 
   377 text {*
   378 text {*
   378   If the input heap file does not have write permission bits set, or
   379   If the input heap file does not have write permission bits set, or
   379   the @{verbatim "-r"} option is given explicitely, then the session
   380   the @{verbatim "-r"} option is given explicitely, then the session
   380   started will be read-only.  That is, the ML world cannot be
   381   started will be read-only.  That is, the ML world cannot be
   409   may happen when errorneous ML code is provided. Also make sure that
   410   may happen when errorneous ML code is provided. Also make sure that
   410   the ML commands are terminated properly by semicolon.
   411   the ML commands are terminated properly by semicolon.
   411 
   412 
   412   \medskip The @{verbatim "-u"} option is a shortcut for @{verbatim
   413   \medskip The @{verbatim "-u"} option is a shortcut for @{verbatim
   413   "-e"} passing ``@{verbatim "use \"ROOT.ML\";"}'' to the ML session.
   414   "-e"} passing ``@{verbatim "use \"ROOT.ML\";"}'' to the ML session.
   414   The @{verbatim "-f"} option passes ``@{verbatim "Session.finish ();"}'',
   415   The @{verbatim "-f"} option passes ``@{verbatim
   415   which is intended mainly for administrative purposes.
   416   "Session.finish();"}'', which is intended mainly for administrative
       
   417   purposes.
   416 
   418 
   417   \medskip The @{verbatim "-m"} option adds identifiers of print modes
   419   \medskip The @{verbatim "-m"} option adds identifiers of print modes
   418   to be made active for this session. Typically, this is used by some
   420   to be made active for this session. Typically, this is used by some
   419   user interface, e.g.\ to enable output of proper mathematical
   421   user interface, e.g.\ to enable output of proper mathematical
   420   symbols.
   422   symbols.
   437   secure by disabling some critical operations, notably runtime
   439   secure by disabling some critical operations, notably runtime
   438   compilation and evaluation of ML source code.
   440   compilation and evaluation of ML source code.
   439 *}
   441 *}
   440 
   442 
   441 
   443 
   442 subsection {* Examples *}
   444 subsubsection {* Examples *}
   443 
   445 
   444 text {*
   446 text {*
   445   Run an interactive session of the default object-logic (as specified
   447   Run an interactive session of the default object-logic (as specified
   446   by the @{setting ISABELLE_LOGIC} setting) like this:
   448   by the @{setting ISABELLE_LOGIC} setting) like this:
   447 \begin{ttbox}
   449 \begin{ttbox}