doc-src/System/Thy/Scala.thy
changeset 48602 342ca8f3197b
parent 47825 4f25960417ae
child 48815 eed6698b2ba0
equal deleted inserted replaced
48601:655b08c2cd89 48602:342ca8f3197b
    12 experimentation within the running application. *}
    12 experimentation within the running application. *}
    13 
    13 
    14 
    14 
    15 section {* Java Runtime Environment within Isabelle \label{sec:tool-java} *}
    15 section {* Java Runtime Environment within Isabelle \label{sec:tool-java} *}
    16 
    16 
    17 text {* The Isabelle @{tool_def java} utility is a direct wrapper for
    17 text {* The @{tool_def java} tool is a direct wrapper for the Java
    18   the Java Runtime Environment, within the regular Isabelle settings
    18   Runtime Environment, within the regular Isabelle settings
    19   environment (\secref{sec:settings}).  The command line arguments are
    19   environment (\secref{sec:settings}).  The command line arguments are
    20   that of the underlying Java version.  It is run in @{verbatim
    20   that of the underlying Java version.  It is run in @{verbatim
    21   "-server"} mode if possible, to improve performance (at the cost of
    21   "-server"} mode if possible, to improve performance (at the cost of
    22   extra startup time).
    22   extra startup time).
    23 
    23 
    36 *}
    36 *}
    37 
    37 
    38 
    38 
    39 section {* Scala toplevel \label{sec:tool-scala} *}
    39 section {* Scala toplevel \label{sec:tool-scala} *}
    40 
    40 
    41 text {* The Isabelle @{tool_def scala} utility is a direct wrapper for
    41 text {* The @{tool_def scala} tool is a direct wrapper for the Scala
    42   the Scala toplevel; see also @{tool java} above.  The command line
    42   toplevel; see also @{tool java} above.  The command line arguments
    43   arguments are that of the underlying Scala version.
    43   are that of the underlying Scala version.
    44 
    44 
    45   This allows to interact with Isabelle/Scala in TTY mode like this:
    45   This allows to interact with Isabelle/Scala in TTY mode like this:
    46 \begin{alltt}
    46 \begin{alltt}
    47   isabelle scala
    47   isabelle scala
    48   scala> isabelle.Isabelle_System.getenv("ISABELLE_HOME")
    48   scala> isabelle.Isabelle_System.getenv("ISABELLE_HOME")
    51 *}
    51 *}
    52 
    52 
    53 
    53 
    54 section {* Scala compiler \label{sec:tool-scalac} *}
    54 section {* Scala compiler \label{sec:tool-scalac} *}
    55 
    55 
    56 text {* The Isabelle @{tool_def scalac} utility is a direct wrapper
    56 text {* The @{tool_def scalac} tool is a direct wrapper for the Scala
    57   for the Scala compiler; see also @{tool scala} above.  The command
    57   compiler; see also @{tool scala} above.  The command line arguments
    58   line arguments are that of the underlying Scala version.
    58   are that of the underlying Scala version.
    59 
    59 
    60   This allows to compile further Scala modules, depending on existing
    60   This allows to compile further Scala modules, depending on existing
    61   Isabelle/Scala functionality.  The resulting class or jar files can
    61   Isabelle/Scala functionality.  The resulting class or jar files can
    62   be added to the @{setting CLASSPATH} via the @{verbatim classpath}
    62   be added to the @{setting CLASSPATH} via the @{verbatim classpath}
    63   Bash function that is provided by the Isabelle process environment.
    63   Bash function that is provided by the Isabelle process environment.