author | wenzelm |
Mon, 06 Apr 2015 12:37:21 +0200 | |
changeset 59929 | a090551e5ec8 |
parent 58618 | 782f0b662cae |
child 61407 | 7ba7b8103565 |
permissions | -rw-r--r-- |
47825 | 1 |
theory Scala |
2 |
imports Base |
|
3 |
begin |
|
4 |
||
58618 | 5 |
chapter \<open>Isabelle/Scala development tools\<close> |
47825 | 6 |
|
58618 | 7 |
text \<open>Isabelle/ML and Isabelle/Scala are the two main language |
47825 | 8 |
environments for Isabelle tool implementations. There are some basic |
9 |
command-line tools to work with the underlying Java Virtual Machine, |
|
10 |
the Scala toplevel and compiler. Note that Isabelle/jEdit |
|
58553 | 11 |
@{cite "isabelle-jedit"} provides a Scala Console for interactive |
58618 | 12 |
experimentation within the running application.\<close> |
47825 | 13 |
|
14 |
||
58618 | 15 |
section \<open>Java Runtime Environment within Isabelle \label{sec:tool-java}\<close> |
47825 | 16 |
|
58618 | 17 |
text \<open>The @{tool_def java} tool is a direct wrapper for the Java |
48602 | 18 |
Runtime Environment, within the regular Isabelle settings |
47825 | 19 |
environment (\secref{sec:settings}). The command line arguments are |
20 |
that of the underlying Java version. It is run in @{verbatim |
|
21 |
"-server"} mode if possible, to improve performance (at the cost of |
|
22 |
extra startup time). |
|
23 |
||
24 |
The @{verbatim java} executable is the one within @{setting |
|
25 |
ISABELLE_JDK_HOME}, according to the standard directory layout for |
|
26 |
official JDK distributions. The class loader is augmented such that |
|
27 |
the name space of @{verbatim "Isabelle/Pure.jar"} is available, |
|
28 |
which is the main Isabelle/Scala module. |
|
29 |
||
30 |
For example, the following command-line invokes the main method of |
|
31 |
class @{verbatim isabelle.GUI_Setup}, which opens a windows with |
|
32 |
some diagnostic information about the Isabelle environment: |
|
33 |
\begin{alltt} |
|
34 |
isabelle java isabelle.GUI_Setup |
|
35 |
\end{alltt} |
|
58618 | 36 |
\<close> |
47825 | 37 |
|
38 |
||
58618 | 39 |
section \<open>Scala toplevel \label{sec:tool-scala}\<close> |
47825 | 40 |
|
58618 | 41 |
text \<open>The @{tool_def scala} tool is a direct wrapper for the Scala |
48602 | 42 |
toplevel; see also @{tool java} above. The command line arguments |
43 |
are that of the underlying Scala version. |
|
47825 | 44 |
|
45 |
This allows to interact with Isabelle/Scala in TTY mode like this: |
|
46 |
\begin{alltt} |
|
47 |
isabelle scala |
|
48 |
scala> isabelle.Isabelle_System.getenv("ISABELLE_HOME") |
|
48815 | 49 |
scala> val options = isabelle.Options.init() |
50 |
scala> options.bool("browser_info") |
|
52116
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
51 |
scala> options.string("document") |
47825 | 52 |
\end{alltt} |
58618 | 53 |
\<close> |
47825 | 54 |
|
55 |
||
58618 | 56 |
section \<open>Scala compiler \label{sec:tool-scalac}\<close> |
47825 | 57 |
|
58618 | 58 |
text \<open>The @{tool_def scalac} tool is a direct wrapper for the Scala |
48602 | 59 |
compiler; see also @{tool scala} above. The command line arguments |
60 |
are that of the underlying Scala version. |
|
47825 | 61 |
|
62 |
This allows to compile further Scala modules, depending on existing |
|
63 |
Isabelle/Scala functionality. The resulting class or jar files can |
|
57855 | 64 |
be added to the Java classpath using the @{verbatim classpath} Bash |
53576
793a429c63e7
maintain classpath in more elementary manner: turn ISABELLE_CLASSPATH into -classpath option, so that all jars are covered by sun.misc.Launcher.AppClassLoader (e.g. relevant for loading add-on resources);
wenzelm
parents:
52116
diff
changeset
|
65 |
function that is provided by the Isabelle process environment. Thus |
793a429c63e7
maintain classpath in more elementary manner: turn ISABELLE_CLASSPATH into -classpath option, so that all jars are covered by sun.misc.Launcher.AppClassLoader (e.g. relevant for loading add-on resources);
wenzelm
parents:
52116
diff
changeset
|
66 |
add-on components can register themselves in a modular manner, see |
793a429c63e7
maintain classpath in more elementary manner: turn ISABELLE_CLASSPATH into -classpath option, so that all jars are covered by sun.misc.Launcher.AppClassLoader (e.g. relevant for loading add-on resources);
wenzelm
parents:
52116
diff
changeset
|
67 |
also \secref{sec:components}. |
47825 | 68 |
|
58553 | 69 |
Note that jEdit @{cite "isabelle-jedit"} has its own mechanisms for |
47825 | 70 |
adding plugin components, which needs special attention since |
58618 | 71 |
it overrides the standard Java class loader.\<close> |
47825 | 72 |
|
52116
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
73 |
|
58618 | 74 |
section \<open>Scala script wrapper\<close> |
52116
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
75 |
|
58618 | 76 |
text \<open>The executable @{executable |
52116
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
77 |
"$ISABELLE_HOME/bin/isabelle_scala_script"} allows to run |
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
78 |
Isabelle/Scala source files stand-alone programs, by using a |
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
79 |
suitable ``hash-bang'' line and executable file permissions. |
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
80 |
|
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
81 |
The subsequent example assumes that the main Isabelle binaries have |
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
82 |
been installed in some directory that is included in @{setting PATH} |
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
83 |
(see also @{tool "install"}): |
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
84 |
|
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
85 |
\begin{alltt} |
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
86 |
#!/usr/bin/env isabelle_scala_script |
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
87 |
|
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
88 |
val options = isabelle.Options.init() |
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
89 |
Console.println("browser_info = " + options.bool("browser_info")) |
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
90 |
Console.println("document = " + options.string("document")) |
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
91 |
\end{alltt} |
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
92 |
|
53982 | 93 |
Alternatively the full @{file |
52116
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
94 |
"$ISABELLE_HOME/bin/isabelle_scala_script"} may be specified in |
58618 | 95 |
expanded form.\<close> |
52116
abf9fcfa65cf
added isabelle_scala_script wrapper -- NB: portable hash-bang allows exactly one executable, without additional arguments;
wenzelm
parents:
48985
diff
changeset
|
96 |
|
47825 | 97 |
end |