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