author | wenzelm |
Sat, 26 Sep 2020 14:29:46 +0200 | |
changeset 72309 | 564012e31db1 |
parent 71579 | 9b49538845cc |
child 72316 | 3cc6aa405858 |
permissions | -rw-r--r-- |
61656 | 1 |
(*:maxLineLen=78:*) |
61575 | 2 |
|
28224 | 3 |
theory Misc |
43564
9864182c6bad
document antiquotations are managed as theory data, with proper name space and entity markup;
wenzelm
parents:
41512
diff
changeset
|
4 |
imports Base |
28224 | 5 |
begin |
6 |
||
58618 | 7 |
chapter \<open>Miscellaneous tools \label{ch:tools}\<close> |
28224 | 8 |
|
58618 | 9 |
text \<open> |
61575 | 10 |
Subsequently we describe various Isabelle related utilities, given in |
11 |
alphabetical order. |
|
58618 | 12 |
\<close> |
28224 | 13 |
|
71579 | 14 |
section \<open>Building Isabelle docker images\<close> |
15 |
||
16 |
text \<open> |
|
17 |
Docker\<^footnote>\<open>\<^url>\<open>https://docs.docker.com\<close>\<close> provides a self-contained environment |
|
18 |
for complex applications called \<^emph>\<open>container\<close>, although it does not fully |
|
19 |
contain the program in a strict sense of the word. This includes basic |
|
20 |
operating system services (usually based on Linux), shared libraries and |
|
21 |
other required packages. Thus Docker is a light-weight alternative to |
|
22 |
regular virtual machines, or a heavy-weight alternative to conventional |
|
23 |
self-contained applications. |
|
24 |
||
25 |
Although Isabelle can be easily run on a variety of OS environments without |
|
26 |
extra containment, Docker images may occasionally be useful when a |
|
27 |
standardized Linux environment is required, even on |
|
28 |
Windows\<^footnote>\<open>\<^url>\<open>https://docs.docker.com/docker-for-windows\<close>\<close> and |
|
29 |
macOS\<^footnote>\<open>\<^url>\<open>https://docs.docker.com/docker-for-mac\<close>\<close>. Further uses are in |
|
30 |
common cloud computing environments, where applications need to be submitted |
|
31 |
as Docker images in the first place. |
|
32 |
||
33 |
\<^medskip> |
|
34 |
The @{tool_def build_docker} tool builds docker images from a standard |
|
35 |
Isabelle application archive for Linux: |
|
36 |
||
37 |
@{verbatim [display] |
|
38 |
\<open>Usage: isabelle build_docker [OPTIONS] APP_ARCHIVE |
|
39 |
||
40 |
Options are: |
|
41 |
-B NAME base image (default "ubuntu") |
|
42 |
-E set bin/isabelle as entrypoint |
|
43 |
-P NAME additional Ubuntu package collection ("X11", "latex") |
|
44 |
-l NAME default logic (default ISABELLE_LOGIC="HOL") |
|
45 |
-n no docker build |
|
46 |
-o FILE output generated Dockerfile |
|
47 |
-p NAME additional Ubuntu package |
|
48 |
-t TAG docker build tag |
|
49 |
-v verbose |
|
50 |
||
51 |
Build Isabelle docker image with default logic image, using a standard |
|
52 |
Isabelle application archive for Linux (local file or remote URL).\<close>} |
|
53 |
||
54 |
Option \<^verbatim>\<open>-E\<close> sets \<^verbatim>\<open>bin/isabelle\<close> of the contained Isabelle distribution as |
|
55 |
the standard entry point of the Docker image. Thus \<^verbatim>\<open>docker run\<close> will |
|
56 |
imitate the \<^verbatim>\<open>isabelle\<close> command-line tool (\secref{sec:isabelle-tool}) of a |
|
57 |
regular local installation, but it lacks proper GUI support: \<^verbatim>\<open>isabelle jedit\<close> |
|
58 |
will not work without further provisions. Note that the default entrypoint |
|
59 |
may be changed later via \<^verbatim>\<open>docker run --entrypoint="..."\<close>. |
|
60 |
||
61 |
Option \<^verbatim>\<open>-t\<close> specifies the Docker image tag: this a symbolic name within the |
|
62 |
local Docker name space, but also relevant for Docker |
|
63 |
Hub\<^footnote>\<open>\<^url>\<open>https://hub.docker.com\<close>\<close>. |
|
64 |
||
65 |
Option \<^verbatim>\<open>-l\<close> specifies the default logic image of the Isabelle distribution |
|
66 |
contained in the Docker environment: it will be produced by \<^verbatim>\<open>isabelle build -b\<close> |
|
67 |
as usual (\secref{sec:tool-build}) and stored within the image. |
|
68 |
||
69 |
\<^medskip> |
|
70 |
Option \<^verbatim>\<open>-B\<close> specifies the Docker image taken as starting point for the |
|
71 |
Isabelle installation: it needs to be a suitable version of Ubuntu Linux. |
|
72 |
The default \<^verbatim>\<open>ubuntu\<close> refers to the latest LTS version provided by Canonical |
|
73 |
as the official Ubuntu vendor\<^footnote>\<open>\<^url>\<open>https://hub.docker.com/_/ubuntu\<close>\<close>. For |
|
74 |
Isabelle2020 this should be Ubuntu 18.04 LTS. |
|
75 |
||
76 |
Option \<^verbatim>\<open>-p\<close> includes additional Ubuntu packages, using the terminology |
|
77 |
of \<^verbatim>\<open>apt-get install\<close> within the underlying Linux distribution. |
|
78 |
||
79 |
Option \<^verbatim>\<open>-P\<close> refers to high-level package collections: \<^verbatim>\<open>X11\<close> or \<^verbatim>\<open>latex\<close> as |
|
80 |
provided by \<^verbatim>\<open>isabelle build_docker\<close> (assuming Ubuntu 18.04 LTS). This |
|
81 |
imposes extra weight on the resulting Docker images. Note that \<^verbatim>\<open>X11\<close> will |
|
82 |
only provide remote X11 support according to the modest GUI quality |
|
83 |
standards of the late 1990-ies. |
|
84 |
||
85 |
\<^medskip> |
|
86 |
Option \<^verbatim>\<open>-n\<close> suppresses the actual \<^verbatim>\<open>docker build\<close> process. Option \<^verbatim>\<open>-o\<close> |
|
87 |
outputs the generated \<^verbatim>\<open>Dockerfile\<close>. Both options together produce a |
|
88 |
Dockerfile only, which might be useful for informative purposes or other |
|
89 |
tools. |
|
90 |
||
91 |
Option \<^verbatim>\<open>-v\<close> disables quiet-mode of the underlying \<^verbatim>\<open>docker build\<close> process. |
|
92 |
\<close> |
|
93 |
||
94 |
||
95 |
subsubsection \<open>Examples\<close> |
|
96 |
||
97 |
text \<open> |
|
98 |
Produce a Dockerfile (without image) from a remote Isabelle distribution: |
|
99 |
@{verbatim [display] |
|
100 |
\<open> isabelle build_docker -E -n -o Dockerfile |
|
101 |
https://isabelle.in.tum.de/website-Isabelle2020/dist/Isabelle2020_linux.tar.gz\<close>} |
|
102 |
||
103 |
Build a standard Isabelle Docker image from a local Isabelle distribution, |
|
104 |
with \<^verbatim>\<open>bin/isabelle\<close> as executable entry point: |
|
105 |
||
106 |
@{verbatim [display] |
|
107 |
\<open> isabelle build_docker -E -t test/isabelle:Isabelle2020 Isabelle2020_linux.tar.gz\<close>} |
|
108 |
||
109 |
Invoke the raw Isabelle/ML process within that image: |
|
110 |
@{verbatim [display] |
|
111 |
\<open> docker run test/isabelle:Isabelle2020 process -e "Session.welcome ()"\<close>} |
|
112 |
||
113 |
Invoke a Linux command-line tool within the contained Isabelle system |
|
114 |
environment: |
|
115 |
@{verbatim [display] |
|
116 |
\<open> docker run test/isabelle:Isabelle2020 env uname -a\<close>} |
|
117 |
The latter should always report a Linux operating system, even when running |
|
118 |
on Windows or macOS. |
|
119 |
\<close> |
|
120 |
||
28224 | 121 |
|
58618 | 122 |
section \<open>Resolving Isabelle components \label{sec:tool-components}\<close> |
48844 | 123 |
|
58618 | 124 |
text \<open> |
48844 | 125 |
The @{tool_def components} tool resolves Isabelle components: |
61407
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
126 |
@{verbatim [display] |
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
127 |
\<open>Usage: isabelle components [OPTIONS] [COMPONENTS ...] |
48844 | 128 |
|
129 |
Options are: |
|
50653
5c85f8b80b95
simplified quick start via "isabelle components -I";
wenzelm
parents:
50132
diff
changeset
|
130 |
-I init user settings |
48844 | 131 |
-R URL component repository |
132 |
(default $ISABELLE_COMPONENT_REPOSITORY) |
|
53435 | 133 |
-a resolve all missing components |
48844 | 134 |
-l list status |
135 |
||
136 |
Resolve Isabelle components via download and installation. |
|
137 |
COMPONENTS are identified via base name. |
|
138 |
||
68224 | 139 |
ISABELLE_COMPONENT_REPOSITORY="https://isabelle.in.tum.de/components"\<close>} |
48844 | 140 |
|
61575 | 141 |
Components are initialized as described in \secref{sec:components} in a |
142 |
permissive manner, which can mark components as ``missing''. This state is |
|
143 |
amended by letting @{tool "components"} download and unpack components that |
|
63680 | 144 |
are published on the default component repository |
68224 | 145 |
\<^url>\<open>https://isabelle.in.tum.de/components\<close> in particular. |
48844 | 146 |
|
61575 | 147 |
Option \<^verbatim>\<open>-R\<close> specifies an alternative component repository. Note that |
148 |
\<^verbatim>\<open>file:///\<close> URLs can be used for local directories. |
|
48844 | 149 |
|
61575 | 150 |
Option \<^verbatim>\<open>-a\<close> selects all missing components to be resolved. Explicit |
151 |
components may be named as command line-arguments as well. Note that |
|
152 |
components are uniquely identified by their base name, while the |
|
153 |
installation takes place in the location that was specified in the attempt |
|
154 |
to initialize the component before. |
|
48844 | 155 |
|
61575 | 156 |
Option \<^verbatim>\<open>-l\<close> lists the current state of available and missing components |
157 |
with their location (full name) within the file-system. |
|
50653
5c85f8b80b95
simplified quick start via "isabelle components -I";
wenzelm
parents:
50132
diff
changeset
|
158 |
|
61575 | 159 |
Option \<^verbatim>\<open>-I\<close> initializes the user settings file to subscribe to the standard |
160 |
components specified in the Isabelle repository clone --- this does not make |
|
161 |
any sense for regular Isabelle releases. If the file already exists, it |
|
162 |
needs to be edited manually according to the printed explanation. |
|
58618 | 163 |
\<close> |
48844 | 164 |
|
165 |
||
58618 | 166 |
section \<open>Viewing documentation \label{sec:tool-doc}\<close> |
28224 | 167 |
|
58618 | 168 |
text \<open> |
52444
2cfe6656d6d6
slightly improved "isabelle doc" based on Isabelle/Scala;
wenzelm
parents:
52052
diff
changeset
|
169 |
The @{tool_def doc} tool displays Isabelle documentation: |
61407
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
170 |
@{verbatim [display] |
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
171 |
\<open>Usage: isabelle doc [DOC ...] |
28224 | 172 |
|
61407
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
173 |
View Isabelle documentation.\<close>} |
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
174 |
|
61575 | 175 |
If called without arguments, it lists all available documents. Each line |
176 |
starts with an identifier, followed by a short description. Any of these |
|
177 |
identifiers may be specified as arguments, in order to display the |
|
72309
564012e31db1
discontinued obsolete DVI document format and related settings/tools;
wenzelm
parents:
71579
diff
changeset
|
178 |
corresponding document. |
28224 | 179 |
|
61406 | 180 |
\<^medskip> |
61575 | 181 |
The @{setting ISABELLE_DOCS} setting specifies the list of directories |
182 |
(separated by colons) to be scanned for documentations. |
|
58618 | 183 |
\<close> |
28224 | 184 |
|
185 |
||
58618 | 186 |
section \<open>Shell commands within the settings environment \label{sec:tool-env}\<close> |
47828 | 187 |
|
61575 | 188 |
text \<open> |
189 |
The @{tool_def env} tool is a direct wrapper for the standard |
|
190 |
\<^verbatim>\<open>/usr/bin/env\<close> command on POSIX systems, running within the Isabelle |
|
191 |
settings environment (\secref{sec:settings}). |
|
47828 | 192 |
|
61575 | 193 |
The command-line arguments are that of the underlying version of \<^verbatim>\<open>env\<close>. For |
194 |
example, the following invokes an instance of the GNU Bash shell within the |
|
195 |
Isabelle environment: |
|
61407
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
196 |
@{verbatim [display] \<open>isabelle env bash\<close>} |
58618 | 197 |
\<close> |
47828 | 198 |
|
199 |
||
58618 | 200 |
section \<open>Inspecting the settings environment \label{sec:tool-getenv}\<close> |
28224 | 201 |
|
58618 | 202 |
text \<open>The Isabelle settings environment --- as provided by the |
28224 | 203 |
site-default and user-specific settings files --- can be inspected |
48602 | 204 |
with the @{tool_def getenv} tool: |
61407
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
205 |
@{verbatim [display] |
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
206 |
\<open>Usage: isabelle getenv [OPTIONS] [VARNAMES ...] |
28224 | 207 |
|
208 |
Options are: |
|
209 |
-a display complete environment |
|
210 |
-b print values only (doesn't work for -a) |
|
31497 | 211 |
-d FILE dump complete environment to FILE |
212 |
(null terminated entries) |
|
28224 | 213 |
|
61407
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
214 |
Get value of VARNAMES from the Isabelle settings.\<close>} |
28224 | 215 |
|
61575 | 216 |
With the \<^verbatim>\<open>-a\<close> option, one may inspect the full process environment that |
217 |
Isabelle related programs are run in. This usually contains much more |
|
218 |
variables than are actually Isabelle settings. Normally, output is a list of |
|
219 |
lines of the form \<open>name\<close>\<^verbatim>\<open>=\<close>\<open>value\<close>. The \<^verbatim>\<open>-b\<close> option causes only the values |
|
220 |
to be printed. |
|
31497 | 221 |
|
61575 | 222 |
Option \<^verbatim>\<open>-d\<close> produces a dump of the complete environment to the specified |
223 |
file. Entries are terminated by the ASCII null character, i.e.\ the C string |
|
224 |
terminator. |
|
58618 | 225 |
\<close> |
28224 | 226 |
|
227 |
||
58618 | 228 |
subsubsection \<open>Examples\<close> |
28224 | 229 |
|
61575 | 230 |
text \<open> |
231 |
Get the location of @{setting ISABELLE_HOME_USER} where user-specific |
|
232 |
information is stored: |
|
61407
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
233 |
@{verbatim [display] \<open>isabelle getenv ISABELLE_HOME_USER\<close>} |
28224 | 234 |
|
61406 | 235 |
\<^medskip> |
61575 | 236 |
Get the value only of the same settings variable, which is particularly |
237 |
useful in shell scripts: |
|
68219 | 238 |
@{verbatim [display] \<open>isabelle getenv -b ISABELLE_HOME_USER\<close>} |
58618 | 239 |
\<close> |
28224 | 240 |
|
241 |
||
71322 | 242 |
section \<open>Mercurial repository setup \label{sec:hg-setup}\<close> |
243 |
||
244 |
text \<open> |
|
245 |
The @{tool_def hg_setup} tool simplifies the setup of Mercurial |
|
71325 | 246 |
repositories, with hosting via Phabricator (\chref{ch:phabricator}) or SSH |
247 |
file server access. |
|
71322 | 248 |
|
249 |
@{verbatim [display] |
|
250 |
\<open>Usage: isabelle hg_setup [OPTIONS] REMOTE LOCAL_DIR |
|
251 |
||
252 |
Options are: |
|
253 |
-n NAME remote repository name (default: base name of LOCAL_DIR) |
|
254 |
-p PATH Mercurial path name (default: "default") |
|
255 |
-r assume that remote repository already exists |
|
256 |
||
257 |
Setup a remote vs. local Mercurial repository: REMOTE either refers to a |
|
258 |
Phabricator server "user@host" or SSH file server "ssh://user@host/path".\<close>} |
|
259 |
||
260 |
The \<^verbatim>\<open>REMOTE\<close> repository specification \<^emph>\<open>excludes\<close> the actual repository |
|
261 |
name: that is given by the base name of \<^verbatim>\<open>LOCAL_DIR\<close>, or via option \<^verbatim>\<open>-n\<close>. |
|
262 |
||
263 |
By default, both sides of the repository are created on demand by default. |
|
264 |
In contrast, option \<^verbatim>\<open>-r\<close> assumes that the remote repository already exists: |
|
265 |
it avoids accidental creation of a persistent repository with unintended |
|
266 |
name. |
|
267 |
||
268 |
The local \<^verbatim>\<open>.hg/hgrc\<close> file is changed to refer to the remote repository, |
|
269 |
usually via the symbolic path name ``\<^verbatim>\<open>default\<close>''; option \<^verbatim>\<open>-p\<close> allows to |
|
270 |
provided a different name. |
|
271 |
\<close> |
|
272 |
||
71324 | 273 |
subsubsection \<open>Examples\<close> |
274 |
||
275 |
text \<open> |
|
276 |
Setup the current directory as a repository with Phabricator server hosting: |
|
277 |
@{verbatim [display] \<open> isabelle hg_setup vcs@vcs.example.org .\<close>} |
|
278 |
||
279 |
\<^medskip> |
|
280 |
Setup the current directory as a repository with plain SSH server hosting: |
|
281 |
@{verbatim [display] \<open> isabelle hg_setup ssh://files.example.org/data/repositories .\<close>} |
|
282 |
||
283 |
\<^medskip> |
|
284 |
Both variants require SSH access to the target server, via public key |
|
285 |
without password. |
|
286 |
\<close> |
|
287 |
||
71322 | 288 |
|
58618 | 289 |
section \<open>Installing standalone Isabelle executables \label{sec:tool-install}\<close> |
28224 | 290 |
|
61575 | 291 |
text \<open> |
292 |
By default, the main Isabelle binaries (@{executable "isabelle"} etc.) are |
|
293 |
just run from their location within the distribution directory, probably |
|
294 |
indirectly by the shell through its @{setting PATH}. Other schemes of |
|
295 |
installation are supported by the @{tool_def install} tool: |
|
61407
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
296 |
@{verbatim [display] |
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
297 |
\<open>Usage: isabelle install [OPTIONS] BINDIR |
28224 | 298 |
|
299 |
Options are: |
|
50132 | 300 |
-d DISTDIR refer to DISTDIR as Isabelle distribution |
28224 | 301 |
(default ISABELLE_HOME) |
302 |
||
50132 | 303 |
Install Isabelle executables with absolute references to the |
61407
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
304 |
distribution directory.\<close>} |
28224 | 305 |
|
61575 | 306 |
The \<^verbatim>\<open>-d\<close> option overrides the current Isabelle distribution directory as |
307 |
determined by @{setting ISABELLE_HOME}. |
|
28224 | 308 |
|
61575 | 309 |
The \<open>BINDIR\<close> argument tells where executable wrapper scripts for |
62588
cd266473b81b
isabelle_process is superseded by "isabelle process" tool;
wenzelm
parents:
62562
diff
changeset
|
310 |
@{executable "isabelle"} and @{executable isabelle_scala_script} should be |
61575 | 311 |
placed, which is typically a directory in the shell's @{setting PATH}, such |
312 |
as \<^verbatim>\<open>$HOME/bin\<close>. |
|
48815 | 313 |
|
61406 | 314 |
\<^medskip> |
61575 | 315 |
It is also possible to make symbolic links of the main Isabelle executables |
316 |
manually, but making separate copies outside the Isabelle distribution |
|
317 |
directory will not work! |
|
318 |
\<close> |
|
28224 | 319 |
|
320 |
||
58618 | 321 |
section \<open>Creating instances of the Isabelle logo\<close> |
28224 | 322 |
|
61575 | 323 |
text \<open> |
324 |
The @{tool_def logo} tool creates instances of the generic Isabelle logo as |
|
325 |
EPS and PDF, for inclusion in {\LaTeX} documents. |
|
61407
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
326 |
@{verbatim [display] |
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
327 |
\<open>Usage: isabelle logo [OPTIONS] XYZ |
28224 | 328 |
|
49072
747835eb2782
"isabelle logo" produces EPS and PDF format simultaneously;
wenzelm
parents:
48985
diff
changeset
|
329 |
Create instance XYZ of the Isabelle logo (as EPS and PDF). |
28224 | 330 |
|
331 |
Options are: |
|
49072
747835eb2782
"isabelle logo" produces EPS and PDF format simultaneously;
wenzelm
parents:
48985
diff
changeset
|
332 |
-n NAME alternative output base name (default "isabelle_xyx") |
61407
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
333 |
-q quiet mode\<close>} |
48936 | 334 |
|
61575 | 335 |
Option \<^verbatim>\<open>-n\<close> specifies an alternative (base) name for the generated files. |
336 |
The default is \<^verbatim>\<open>isabelle_\<close>\<open>xyz\<close> in lower-case. |
|
48936 | 337 |
|
61503 | 338 |
Option \<^verbatim>\<open>-q\<close> omits printing of the result file name. |
48936 | 339 |
|
61406 | 340 |
\<^medskip> |
61575 | 341 |
Implementors of Isabelle tools and applications are encouraged to make |
342 |
derived Isabelle logos for their own projects using this template. |
|
343 |
\<close> |
|
28224 | 344 |
|
345 |
||
58618 | 346 |
section \<open>Output the version identifier of the Isabelle distribution\<close> |
28224 | 347 |
|
58618 | 348 |
text \<open> |
48602 | 349 |
The @{tool_def version} tool displays Isabelle version information: |
61407
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
350 |
@{verbatim [display] |
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
351 |
\<open>Usage: isabelle version [OPTIONS] |
41511 | 352 |
|
353 |
Options are: |
|
354 |
-i short identification (derived from Mercurial id) |
|
355 |
||
61407
7ba7b8103565
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61406
diff
changeset
|
356 |
Display Isabelle version information.\<close>} |
41511 | 357 |
|
61406 | 358 |
\<^medskip> |
61575 | 359 |
The default is to output the full version string of the Isabelle |
71578 | 360 |
distribution, e.g.\ ``\<^verbatim>\<open>Isabelle2020: April 2020\<close>. |
41511 | 361 |
|
61575 | 362 |
The \<^verbatim>\<open>-i\<close> option produces a short identification derived from the Mercurial |
363 |
id of the @{setting ISABELLE_HOME} directory. |
|
58618 | 364 |
\<close> |
28224 | 365 |
|
67399 | 366 |
end |