author | wenzelm |
Tue, 20 Oct 2015 23:53:40 +0200 | |
changeset 61493 | 0debd22f0c0e |
parent 61483 | 07c8d5d8acab |
child 61503 | 28e788ca2c5d |
permissions | -rw-r--r-- |
53981 | 1 |
(*:wrap=hard:maxLineLen=78:*) |
2 |
||
53769 | 3 |
theory JEdit |
4 |
imports Base |
|
5 |
begin |
|
6 |
||
58618 | 7 |
chapter \<open>Introduction\<close> |
53769 | 8 |
|
58618 | 9 |
section \<open>Concepts and terminology\<close> |
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
10 |
|
58618 | 11 |
text \<open> |
61477 | 12 |
Isabelle/jEdit is a Prover IDE that integrates \<^emph>\<open>parallel proof |
13 |
checking\<close> @{cite "Wenzel:2009" and "Wenzel:2013:ITP"} with |
|
14 |
\<^emph>\<open>asynchronous user interaction\<close> @{cite "Wenzel:2010" and |
|
58556 | 15 |
"Wenzel:2012:UITP-EPTCS" and "Wenzel:2014:ITP-PIDE" and "Wenzel:2014:UITP"}, |
61477 | 16 |
based on a document-oriented approach to \<^emph>\<open>continuous proof processing\<close> |
58556 | 17 |
@{cite "Wenzel:2011:CICM" and "Wenzel:2012"}. Many concepts and system |
18 |
components are fit together in order to make this work. The main building |
|
19 |
blocks are as follows. |
|
53769 | 20 |
|
61439 | 21 |
\<^descr>[PIDE] is a general framework for Prover IDEs based on Isabelle/Scala. |
57310 | 22 |
It is built around a concept of parallel and asynchronous document |
23 |
processing, which is supported natively by the parallel proof engine that is |
|
24 |
implemented in Isabelle/ML. The traditional prover command loop is given up; |
|
25 |
instead there is direct support for editing of source text, with rich formal |
|
26 |
markup for GUI rendering. |
|
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
27 |
|
61439 | 28 |
\<^descr>[Isabelle/ML] is the implementation and extension language of |
58554 | 29 |
Isabelle, see also @{cite "isabelle-implementation"}. It is integrated |
54329 | 30 |
into the logical context of Isabelle/Isar and allows to manipulate |
31 |
logical entities directly. Arbitrary add-on tools may be implemented |
|
32 |
for object-logics such as Isabelle/HOL. |
|
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
33 |
|
61439 | 34 |
\<^descr>[Isabelle/Scala] is the system programming language of |
54321 | 35 |
Isabelle. It extends the pure logical environment of Isabelle/ML |
36 |
towards the ``real world'' of graphical user interfaces, text |
|
37 |
editors, IDE frameworks, web services etc. Special infrastructure |
|
54372 | 38 |
allows to transfer algebraic datatypes and formatted text easily |
39 |
between ML and Scala, using asynchronous protocol commands. |
|
54321 | 40 |
|
61439 | 41 |
\<^descr>[jEdit] is a sophisticated text editor implemented in |
54703 | 42 |
Java.\footnote{@{url "http://www.jedit.org"}} It is easily extensible |
54329 | 43 |
by plugins written in languages that work on the JVM, e.g.\ |
57337 | 44 |
Scala\footnote{@{url "http://www.scala-lang.org"}}. |
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
45 |
|
61439 | 46 |
\<^descr>[Isabelle/jEdit] is the main example application of the PIDE |
54329 | 47 |
framework and the default user-interface for Isabelle. It targets |
48 |
both beginners and experts. Technically, Isabelle/jEdit combines a |
|
54372 | 49 |
slightly modified version of the jEdit code base with a special |
50 |
plugin for Isabelle, integrated as standalone application for the |
|
51 |
main operating system platforms: Linux, Windows, Mac OS X. |
|
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
52 |
|
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
53 |
|
54321 | 54 |
The subtle differences of Isabelle/ML versus Standard ML, |
54330 | 55 |
Isabelle/Scala versus Scala, Isabelle/jEdit versus jEdit need to be |
56 |
taken into account when discussing any of these PIDE building blocks |
|
57 |
in public forums, mailing lists, or even scientific publications. |
|
58618 | 58 |
\<close> |
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
59 |
|
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
60 |
|
58618 | 61 |
section \<open>The Isabelle/jEdit Prover IDE\<close> |
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
62 |
|
58618 | 63 |
text \<open> |
54357 | 64 |
\begin{figure}[htb] |
54331 | 65 |
\begin{center} |
57312 | 66 |
\includegraphics[scale=0.333]{isabelle-jedit} |
54331 | 67 |
\end{center} |
68 |
\caption{The Isabelle/jEdit Prover IDE} |
|
54357 | 69 |
\label{fig:isabelle-jedit} |
54331 | 70 |
\end{figure} |
53773 | 71 |
|
57337 | 72 |
Isabelle/jEdit (\figref{fig:isabelle-jedit}) consists of some plugins for |
73 |
the jEdit text editor, while preserving its general look-and-feel as far as |
|
74 |
possible. The main plugin is called ``Isabelle'' and has its own menu |
|
61477 | 75 |
\<^emph>\<open>Plugins~/ Isabelle\<close> with access to several panels (see also |
76 |
\secref{sec:dockables}), as well as \<^emph>\<open>Plugins~/ Plugin Options~/ |
|
77 |
Isabelle\<close> (see also \secref{sec:options}). |
|
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
78 |
|
57337 | 79 |
The options allow to specify a logic session name --- the same selector is |
61477 | 80 |
accessible in the \<^emph>\<open>Theories\<close> panel (\secref{sec:theories}). On |
57337 | 81 |
application startup, the selected logic session image is provided |
60270 | 82 |
automatically by the Isabelle build tool @{cite "isabelle-system"}: if it is |
57337 | 83 |
absent or outdated wrt.\ its sources, the build process updates it before |
60257 | 84 |
entering the Prover IDE. Change of the logic session within Isabelle/jEdit |
57420 | 85 |
requires a restart of the whole application. |
53769 | 86 |
|
61415 | 87 |
\<^medskip> |
88 |
The main job of the Prover IDE is to manage sources and their |
|
57337 | 89 |
changes, taking the logical structure as a formal document into account (see |
90 |
also \secref{sec:document-model}). The editor and the prover are connected |
|
91 |
asynchronously in a lock-free manner. The prover is free to organize the |
|
92 |
checking of the formal text in parallel on multiple cores, and provides |
|
93 |
feedback via markup, which is rendered in the editor via colors, boxes, |
|
57420 | 94 |
squiggly underlines, hyperlinks, popup windows, icons, clickable output etc. |
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
95 |
|
57337 | 96 |
Using the mouse together with the modifier key @{verbatim CONTROL} (Linux, |
97 |
Windows) or @{verbatim COMMAND} (Mac OS X) exposes additional formal content |
|
98 |
via tooltips and/or hyperlinks (see also \secref{sec:tooltips-hyperlinks}). |
|
57420 | 99 |
Output (in popups etc.) may be explored recursively, using the same |
57337 | 100 |
techniques as in the editor source buffer. |
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
101 |
|
57337 | 102 |
Thus the Prover IDE gives an impression of direct access to formal content |
103 |
of the prover within the editor, but in reality only certain aspects are |
|
60257 | 104 |
exposed, according to the possibilities of the prover and its many add-on |
105 |
tools. |
|
58618 | 106 |
\<close> |
53769 | 107 |
|
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
108 |
|
58618 | 109 |
subsection \<open>Documentation\<close> |
54321 | 110 |
|
58618 | 111 |
text \<open> |
61477 | 112 |
The \<^emph>\<open>Documentation\<close> panel of Isabelle/jEdit provides access to the |
57310 | 113 |
standard Isabelle documentation: PDF files are opened by regular desktop |
57338 | 114 |
operations of the underlying platform. The section ``Original jEdit |
61477 | 115 |
Documentation'' contains the original \<^emph>\<open>User's Guide\<close> of this |
57338 | 116 |
sophisticated text editor. The same is accessible via the @{verbatim Help} |
117 |
menu or @{verbatim F1} keyboard shortcut, using the built-in HTML viewer of |
|
61477 | 118 |
Java/Swing. The latter also includes \<^emph>\<open>Frequently Asked Questions\<close> and |
57338 | 119 |
documentation of individual plugins. |
54321 | 120 |
|
57310 | 121 |
Most of the information about generic jEdit is relevant for Isabelle/jEdit |
122 |
as well, but one needs to keep in mind that defaults sometimes differ, and |
|
123 |
the official jEdit documentation does not know about the Isabelle plugin |
|
124 |
with its support for continuous checking of formal source text: jEdit is a |
|
125 |
plain text editor, but Isabelle/jEdit is a Prover IDE. |
|
58618 | 126 |
\<close> |
54321 | 127 |
|
128 |
||
58618 | 129 |
subsection \<open>Plugins\<close> |
54321 | 130 |
|
58618 | 131 |
text \<open> |
61477 | 132 |
The \<^emph>\<open>Plugin Manager\<close> of jEdit allows to augment editor functionality by |
57420 | 133 |
JVM modules (jars) that are provided by the central plugin repository, which |
134 |
is accessible via various mirror sites. |
|
54321 | 135 |
|
57420 | 136 |
Connecting to the plugin server-infrastructure of the jEdit project allows |
137 |
to update bundled plugins or to add further functionality. This needs to be |
|
138 |
done with the usual care for such an open bazaar of contributions. Arbitrary |
|
139 |
combinations of add-on features are apt to cause problems. It is advisable |
|
140 |
to start with the default configuration of Isabelle/jEdit and develop some |
|
141 |
understanding how it is supposed to work, before loading additional plugins |
|
142 |
at a grand scale. |
|
54321 | 143 |
|
61415 | 144 |
\<^medskip> |
61477 | 145 |
The main \<^emph>\<open>Isabelle\<close> plugin is an integral part of |
57310 | 146 |
Isabelle/jEdit and needs to remain active at all times! A few additional |
147 |
plugins are bundled with Isabelle/jEdit for convenience or out of necessity, |
|
61477 | 148 |
notably \<^emph>\<open>Console\<close> with its Isabelle/Scala sub-plugin |
149 |
(\secref{sec:scala-console}) and \<^emph>\<open>SideKick\<close> with some Isabelle-specific |
|
57310 | 150 |
parsers for document tree structure (\secref{sec:sidekick}). The |
61477 | 151 |
\<^emph>\<open>Navigator\<close> plugin is particularly important for hyperlinks within the |
57310 | 152 |
formal document-model (\secref{sec:tooltips-hyperlinks}). Further plugins |
61477 | 153 |
(e.g.\ \<^emph>\<open>ErrorList\<close>, \<^emph>\<open>Code2HTML\<close>) are included to saturate the |
57310 | 154 |
dependencies of bundled plugins, but have no particular use in |
57420 | 155 |
Isabelle/jEdit. |
58618 | 156 |
\<close> |
54321 | 157 |
|
158 |
||
58618 | 159 |
subsection \<open>Options \label{sec:options}\<close> |
54321 | 160 |
|
58618 | 161 |
text \<open>Both jEdit and Isabelle have distinctive management of |
54348 | 162 |
persistent options. |
54321 | 163 |
|
61477 | 164 |
Regular jEdit options are accessible via the dialogs \<^emph>\<open>Utilities~/ |
165 |
Global Options\<close> or \<^emph>\<open>Plugins~/ Plugin Options\<close>, with a second chance to |
|
57310 | 166 |
flip the two within the central options dialog. Changes are stored in |
167 |
@{file_unchecked "$ISABELLE_HOME_USER/jedit/properties"} and |
|
168 |
@{file_unchecked "$ISABELLE_HOME_USER/jedit/keymaps"}. |
|
169 |
||
170 |
Isabelle system options are managed by Isabelle/Scala and changes are stored |
|
171 |
in @{file_unchecked "$ISABELLE_HOME_USER/etc/preferences"}, independently of |
|
60270 | 172 |
other jEdit properties. See also @{cite "isabelle-system"}, especially the |
57310 | 173 |
coverage of sessions and command-line tools like @{tool build} or @{tool |
54372 | 174 |
options}. |
54321 | 175 |
|
61477 | 176 |
Those Isabelle options that are declared as \<^bold>\<open>public\<close> are configurable |
177 |
in Isabelle/jEdit via \<^emph>\<open>Plugin Options~/ Isabelle~/ General\<close>. Moreover, |
|
57310 | 178 |
there are various options for rendering of document content, which are |
61477 | 179 |
configurable via \<^emph>\<open>Plugin Options~/ Isabelle~/ Rendering\<close>. Thus |
180 |
\<^emph>\<open>Plugin Options~/ Isabelle\<close> in jEdit provides a view on a subset of |
|
57310 | 181 |
Isabelle system options. Note that some of these options affect general |
182 |
parameters that are relevant outside Isabelle/jEdit as well, e.g.\ |
|
183 |
@{system_option threads} or @{system_option parallel_proofs} for the |
|
60270 | 184 |
Isabelle build tool @{cite "isabelle-system"}, but it is possible to use the |
57310 | 185 |
settings variable @{setting ISABELLE_BUILD_OPTIONS} to change defaults for |
186 |
batch builds without affecting Isabelle/jEdit. |
|
54329 | 187 |
|
57627
65fc7ae1bf66
added action "isabelle.options" (despite problems with initial window size);
wenzelm
parents:
57603
diff
changeset
|
188 |
The jEdit action @{action_def isabelle.options} opens the options dialog for |
65fc7ae1bf66
added action "isabelle.options" (despite problems with initial window size);
wenzelm
parents:
57603
diff
changeset
|
189 |
the Isabelle plugin; it can be mapped to editor GUI elements as usual. |
65fc7ae1bf66
added action "isabelle.options" (despite problems with initial window size);
wenzelm
parents:
57603
diff
changeset
|
190 |
|
61415 | 191 |
\<^medskip> |
192 |
Options are usually loaded on startup and saved on shutdown of |
|
57310 | 193 |
Isabelle/jEdit. Editing the machine-generated @{file_unchecked |
54372 | 194 |
"$ISABELLE_HOME_USER/jedit/properties"} or @{file_unchecked |
57310 | 195 |
"$ISABELLE_HOME_USER/etc/preferences"} manually while the application is |
58618 | 196 |
running is likely to cause surprise due to lost update!\<close> |
54321 | 197 |
|
198 |
||
58618 | 199 |
subsection \<open>Keymaps\<close> |
54321 | 200 |
|
58618 | 201 |
text \<open>Keyboard shortcuts used to be managed as jEdit properties in |
54321 | 202 |
the past, but recent versions (2013) have a separate concept of |
61477 | 203 |
\<^emph>\<open>keymap\<close> that is configurable via \<^emph>\<open>Global Options~/ |
204 |
Shortcuts\<close>. The @{verbatim imported} keymap is derived from the |
|
54330 | 205 |
initial environment of properties that is available at the first |
54348 | 206 |
start of the editor; afterwards the keymap file takes precedence. |
54321 | 207 |
|
57310 | 208 |
This is relevant for Isabelle/jEdit due to various fine-tuning of default |
209 |
properties, and additional keyboard shortcuts for Isabelle-specific |
|
210 |
functionality. Users may change their keymap later, but need to copy some |
|
57335 | 211 |
keyboard shortcuts manually (see also @{file_unchecked |
57420 | 212 |
"$ISABELLE_HOME_USER/jedit/keymaps"} versus @{verbatim shortcut} properties |
213 |
in @{file "$ISABELLE_HOME/src/Tools/jEdit/src/jEdit.props"}). |
|
58618 | 214 |
\<close> |
54321 | 215 |
|
216 |
||
58618 | 217 |
section \<open>Command-line invocation \label{sec:command-line}\<close> |
57320
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
218 |
|
58618 | 219 |
text \<open> |
57320
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
220 |
Isabelle/jEdit is normally invoked as standalone application, with |
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
221 |
platform-specific executable wrappers for Linux, Windows, Mac OS X. |
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
222 |
Nonetheless it is occasionally useful to invoke the Prover IDE on the |
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
223 |
command-line, with some extra options and environment settings as explained |
57329 | 224 |
below. The command-line usage of @{tool_def jedit} is as follows: |
61408
9020a3ba6c9a
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61199
diff
changeset
|
225 |
@{verbatim [display] |
9020a3ba6c9a
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61199
diff
changeset
|
226 |
\<open>Usage: isabelle jedit [OPTIONS] [FILES ...] |
57320
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
227 |
|
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
228 |
Options are: |
61132 | 229 |
-J OPTION add JVM runtime option |
57320
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
230 |
-b build only |
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
231 |
-d DIR include session directory |
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
232 |
-f fresh build |
61132 | 233 |
-j OPTION add jEdit runtime option |
234 |
-l NAME logic image name |
|
57320
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
235 |
-m MODE add print mode for output |
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
236 |
-n no build of session image on startup |
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
237 |
-s system build mode for session image |
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
238 |
|
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
239 |
Start jEdit with Isabelle plugin setup and open theory FILES |
61408
9020a3ba6c9a
@{verbatim [display]} supersedes old alltt/ttbox;
wenzelm
parents:
61199
diff
changeset
|
240 |
(default "$USER_HOME/Scratch.thy").\<close>} |
57320
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
241 |
|
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
242 |
The @{verbatim "-l"} option specifies the session name of the logic |
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
243 |
image to be used for proof processing. Additional session root |
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
244 |
directories may be included via option @{verbatim "-d"} to augment |
60270 | 245 |
that name space of @{tool build} @{cite "isabelle-system"}. |
57320
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
246 |
|
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
247 |
By default, the specified image is checked and built on demand. The |
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
248 |
@{verbatim "-s"} option determines where to store the result session image |
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
249 |
of @{tool build}. The @{verbatim "-n"} option bypasses the implicit build |
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
250 |
process for the selected session image. |
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
251 |
|
57420 | 252 |
The @{verbatim "-m"} option specifies additional print modes for the prover |
253 |
process. Note that the system option @{system_option_ref jedit_print_mode} |
|
61477 | 254 |
allows to do the same persistently (e.g.\ via the \<^emph>\<open>Plugin Options\<close> |
57420 | 255 |
dialog of Isabelle/jEdit), without requiring command-line invocation. |
57320
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
256 |
|
57420 | 257 |
The @{verbatim "-J"} and @{verbatim "-j"} options allow to pass additional |
258 |
low-level options to the JVM or jEdit, respectively. The defaults are |
|
60270 | 259 |
provided by the Isabelle settings environment @{cite "isabelle-system"}, but |
58554 | 260 |
note that these only work for the command-line tool described here, and not |
261 |
the regular application. |
|
57320
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
262 |
|
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
263 |
The @{verbatim "-b"} and @{verbatim "-f"} options control the self-build |
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
264 |
mechanism of Isabelle/jEdit. This is only relevant for building from |
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
265 |
sources, which also requires an auxiliary @{verbatim jedit_build} component |
57420 | 266 |
from @{url "http://isabelle.in.tum.de/components"}. The official |
267 |
Isabelle release already includes a pre-built version of Isabelle/jEdit. |
|
58618 | 268 |
\<close> |
57320
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
269 |
|
00f2c8d1aa0b
more on command-line invocation -- moved material from system manual;
wenzelm
parents:
57319
diff
changeset
|
270 |
|
58618 | 271 |
chapter \<open>Augmented jEdit functionality\<close> |
57318 | 272 |
|
60291 | 273 |
section \<open>GUI rendering\<close> |
274 |
||
275 |
subsection \<open>Look-and-feel \label{sec:look-and-feel}\<close> |
|
54321 | 276 |
|
60291 | 277 |
text \<open> |
278 |
jEdit is a Java/AWT/Swing application with some ambition to support |
|
279 |
``native'' look-and-feel on all platforms, within the limits of what Oracle |
|
280 |
as Java provider and major operating system distributors allow (see also |
|
281 |
\secref{sec:problems}). |
|
54321 | 282 |
|
54329 | 283 |
Isabelle/jEdit enables platform-specific look-and-feel by default as |
57420 | 284 |
follows. |
54321 | 285 |
|
61477 | 286 |
\<^descr>[Linux:] The platform-independent \<^emph>\<open>Nimbus\<close> is used by |
54372 | 287 |
default. |
54321 | 288 |
|
61477 | 289 |
\<^emph>\<open>GTK+\<close> also works under the side-condition that the overall GTK theme |
60256 | 290 |
is selected in a Swing-friendly way.\footnote{GTK support in Java/Swing was |
291 |
once marketed aggressively by Sun, but never quite finished. Today (2015) it |
|
57310 | 292 |
is lagging behind further development of Swing and GTK. The graphics |
60256 | 293 |
rendering performance can be worse than for other Swing look-and-feels. |
294 |
Nonetheless it has its uses for displays with very high resolution (such as |
|
295 |
``4K'' or ``UHD'' models), because the rendering by the external library is |
|
296 |
subject to global system settings for font scaling.} |
|
54321 | 297 |
|
61477 | 298 |
\<^descr>[Windows:] Regular \<^emph>\<open>Windows\<close> is used by default, but |
299 |
\<^emph>\<open>Windows Classic\<close> also works. |
|
54372 | 300 |
|
61477 | 301 |
\<^descr>[Mac OS X:] Regular \<^emph>\<open>Mac OS X\<close> is used by default. |
54372 | 302 |
|
61477 | 303 |
The bundled \<^emph>\<open>MacOSX\<close> plugin provides various functions that are |
57420 | 304 |
expected from applications on that particular platform: quit from menu or |
305 |
dock, preferences menu, drag-and-drop of text files on the application, |
|
57310 | 306 |
full-screen mode for main editor windows. It is advisable to have the |
61477 | 307 |
\<^emph>\<open>MacOSX\<close> plugin enabled all the time on that platform. |
54321 | 308 |
|
309 |
||
310 |
Users may experiment with different look-and-feels, but need to keep |
|
54329 | 311 |
in mind that this extra variance of GUI functionality is unlikely to |
54372 | 312 |
work in arbitrary combinations. The platform-independent |
61477 | 313 |
\<^emph>\<open>Nimbus\<close> and \<^emph>\<open>Metal\<close> should always work. The historic |
314 |
\<^emph>\<open>CDE/Motif\<close> should be ignored. |
|
54372 | 315 |
|
61477 | 316 |
After changing the look-and-feel in \<^emph>\<open>Global Options~/ |
317 |
Appearance\<close>, it is advisable to restart Isabelle/jEdit in order to |
|
60291 | 318 |
take full effect. |
319 |
\<close> |
|
320 |
||
321 |
||
322 |
subsection \<open>Displays with very high resolution \label{sec:hdpi}\<close> |
|
323 |
||
324 |
text \<open> |
|
325 |
Many years ago, displays with $1024 \times 768$ or $1280 \times 1024$ pixels |
|
326 |
were considered ``high resolution'' and bitmap fonts with 12 or 14 pixels as |
|
327 |
adequate for text rendering. Today (2015), we routinely see ``Full HD'' |
|
328 |
monitors at $1920 \times 1080$ pixels, and occasionally ``Ultra HD'' at |
|
329 |
$3840 \times 2160$ or more, but GUI rendering did not really progress |
|
330 |
beyond the old standards. |
|
331 |
||
332 |
Isabelle/jEdit defaults are a compromise for reasonable out-of-the box |
|
333 |
results on common platforms and medium resolution displays (e.g.\ the ``Full |
|
334 |
HD'' category). Subsequently there are further hints to improve on that. |
|
335 |
||
61415 | 336 |
\<^medskip> |
61477 | 337 |
The \<^bold>\<open>operating-system platform\<close> usually provides some |
60291 | 338 |
configuration for global scaling of text fonts, e.g.\ $120\%$--$250\%$ on |
339 |
Windows. Changing that only has a partial effect on GUI rendering; |
|
340 |
satisfactory display quality requires further adjustments. |
|
341 |
||
61415 | 342 |
\<^medskip> |
61477 | 343 |
The Isabelle/jEdit \<^bold>\<open>application\<close> and its plugins provide |
60291 | 344 |
various font properties that are summarized below. |
345 |
||
61477 | 346 |
\<^item> \<^emph>\<open>Global Options / Text Area / Text font\<close>: the main text area |
60291 | 347 |
font, which is also used as reference point for various derived font sizes, |
348 |
e.g.\ the Output panel (\secref{sec:output}). |
|
349 |
||
61477 | 350 |
\<^item> \<^emph>\<open>Global Options / Gutter / Gutter font\<close>: the font for the gutter |
60291 | 351 |
area left of the main text area, e.g.\ relevant for display of line numbers |
352 |
(disabled by default). |
|
353 |
||
61477 | 354 |
\<^item> \<^emph>\<open>Global Options / Appearance / Button, menu and label font\<close> as |
355 |
well as \<^emph>\<open>List and text field font\<close>: this specifies the primary and |
|
356 |
secondary font for the old \<^emph>\<open>Metal\<close> look-and-feel |
|
60291 | 357 |
(\secref{sec:look-and-feel}), which happens to scale better than newer ones |
61477 | 358 |
like \<^emph>\<open>Nimbus\<close>. |
60291 | 359 |
|
61477 | 360 |
\<^item> \<^emph>\<open>Plugin Options / Isabelle / General / Reset Font Size\<close>: the main |
60291 | 361 |
text area font size for action @{action_ref "isabelle.reset-font-size"}, |
362 |
e.g.\ relevant for quick scaling like in major web browsers. |
|
363 |
||
61477 | 364 |
\<^item> \<^emph>\<open>Plugin Options / Console / General / Font\<close>: the console window |
60291 | 365 |
font, e.g.\ relevant for Isabelle/Scala command-line. |
366 |
||
367 |
||
61477 | 368 |
In \figref{fig:isabelle-jedit-hdpi} the \<^emph>\<open>Metal\<close> look-and-feel is |
60291 | 369 |
configured with custom fonts at 30 pixels, and the main text area and |
61477 | 370 |
console at 36 pixels. Despite the old-fashioned appearance of \<^emph>\<open>Metal\<close>, |
60291 | 371 |
this leads to decent rendering quality on all platforms. |
372 |
||
373 |
\begin{figure}[htb] |
|
374 |
\begin{center} |
|
375 |
\includegraphics[width=\textwidth]{isabelle-jedit-hdpi} |
|
376 |
\end{center} |
|
377 |
\caption{Metal look-and-feel with custom fonts for very high resolution} |
|
378 |
\label{fig:isabelle-jedit-hdpi} |
|
379 |
\end{figure} |
|
380 |
||
61477 | 381 |
On Linux, it is also possible to use \<^emph>\<open>GTK+\<close> with a suitable theme and |
60291 | 382 |
global font scaling. On Mac OS X, the default setup for ``Retina'' displays |
383 |
should work adequately with the native look-and-feel. |
|
384 |
\<close> |
|
54321 | 385 |
|
386 |
||
58618 | 387 |
section \<open>Dockable windows \label{sec:dockables}\<close> |
57316 | 388 |
|
58618 | 389 |
text \<open> |
61477 | 390 |
In jEdit terminology, a \<^emph>\<open>view\<close> is an editor window with one or more |
391 |
\<^emph>\<open>text areas\<close> that show the content of one or more \<^emph>\<open>buffers\<close>. A |
|
392 |
regular view may be surrounded by \<^emph>\<open>dockable windows\<close> that show |
|
393 |
additional information in arbitrary format, not just text; a \<^emph>\<open>plain |
|
394 |
view\<close> does not allow dockables. The \<^emph>\<open>dockable window manager\<close> of jEdit |
|
395 |
organizes these dockable windows, either as \<^emph>\<open>floating\<close> windows, or |
|
396 |
\<^emph>\<open>docked\<close> panels within one of the four margins of the view. There may |
|
57316 | 397 |
be any number of floating instances of some dockable window, but at most one |
61477 | 398 |
docked instance; jEdit actions that address \<^emph>\<open>the\<close> dockable window of a |
57316 | 399 |
particular kind refer to the unique docked instance. |
400 |
||
401 |
Dockables are used routinely in jEdit for important functionality like |
|
61477 | 402 |
\<^emph>\<open>HyperSearch Results\<close> or the \<^emph>\<open>File System Browser\<close>. Plugins often |
57316 | 403 |
provide a central dockable to access their key functionality, which may be |
404 |
opened by the user on demand. The Isabelle/jEdit plugin takes this approach |
|
60257 | 405 |
to the extreme: its plugin menu provides the entry-points to many panels |
406 |
that are managed as dockable windows. Some important panels are docked by |
|
61477 | 407 |
default, e.g.\ \<^emph>\<open>Documentation\<close>, \<^emph>\<open>Output\<close>, \<^emph>\<open>Query\<close>, but the |
60257 | 408 |
user can change this arrangement easily and persistently. |
57316 | 409 |
|
410 |
Compared to plain jEdit, dockable window management in Isabelle/jEdit is |
|
411 |
slightly augmented according to the the following principles: |
|
412 |
||
61477 | 413 |
\<^item> Floating windows are dependent on the main window as \<^emph>\<open>dialog\<close> in |
57316 | 414 |
the sense of Java/AWT/Swing. Dialog windows always stay on top of the view, |
415 |
which is particularly important in full-screen mode. The desktop environment |
|
416 |
of the underlying platform may impose further policies on such dependent |
|
417 |
dialogs, in contrast to fully independent windows, e.g.\ some window |
|
418 |
management functions may be missing. |
|
419 |
||
61415 | 420 |
\<^item> Keyboard focus of the main view vs.\ a dockable window is carefully |
57316 | 421 |
managed according to the intended semantics, as a panel mainly for output or |
61477 | 422 |
input. For example, activating the \<^emph>\<open>Output\<close> (\secref{sec:output}) panel |
57316 | 423 |
via the dockable window manager returns keyboard focus to the main text |
61477 | 424 |
area, but for \<^emph>\<open>Query\<close> (\secref{sec:query}) the focus is given to the |
57316 | 425 |
main input field of that panel. |
426 |
||
61415 | 427 |
\<^item> Panels that provide their own text area for output have an additional |
61477 | 428 |
dockable menu item \<^emph>\<open>Detach\<close>. This produces an independent copy of the |
429 |
current output as a floating \<^emph>\<open>Info\<close> window, which displays that content |
|
57316 | 430 |
independently of ongoing changes of the PIDE document-model. Note that |
431 |
Isabelle/jEdit popup windows (\secref{sec:tooltips-hyperlinks}) provide a |
|
61477 | 432 |
similar \<^emph>\<open>Detach\<close> operation as an icon. |
58618 | 433 |
\<close> |
57316 | 434 |
|
435 |
||
58618 | 436 |
section \<open>Isabelle symbols \label{sec:symbols}\<close> |
57319 | 437 |
|
58618 | 438 |
text \<open> |
61477 | 439 |
Isabelle sources consist of \<^emph>\<open>symbols\<close> that extend plain ASCII to allow |
57420 | 440 |
infinitely many mathematical symbols within the formal sources. This works |
441 |
without depending on particular encodings and varying Unicode |
|
442 |
standards.\footnote{Raw Unicode characters within formal sources would |
|
443 |
compromise portability and reliability in the face of changing |
|
444 |
interpretation of special features of Unicode, such as Combining Characters |
|
58554 | 445 |
or Bi-directional Text.} See also @{cite "Wenzel:2011:CICM"}. |
57319 | 446 |
|
57420 | 447 |
For the prover back-end, formal text consists of ASCII characters that are |
448 |
grouped according to some simple rules, e.g.\ as plain ``@{verbatim a}'' or |
|
449 |
symbolic ``@{verbatim "\<alpha>"}''. For the editor front-end, a certain subset of |
|
450 |
symbols is rendered physically via Unicode glyphs, in order to show |
|
61493 | 451 |
``@{verbatim "\<alpha>"}'' as ``\<open>\<alpha>\<close>'', for example. This symbol |
57420 | 452 |
interpretation is specified by the Isabelle system distribution in @{file |
57319 | 453 |
"$ISABELLE_HOME/etc/symbols"} and may be augmented by the user in |
454 |
@{file_unchecked "$ISABELLE_HOME_USER/etc/symbols"}. |
|
455 |
||
58554 | 456 |
The appendix of @{cite "isabelle-isar-ref"} gives an overview of the |
57319 | 457 |
standard interpretation of finitely many symbols from the infinite |
58554 | 458 |
collection. Uninterpreted symbols are displayed literally, e.g.\ |
459 |
``@{verbatim "\<foobar>"}''. Overlap of Unicode characters used in symbol |
|
460 |
interpretation with informal ones (which might appear e.g.\ in comments) |
|
461 |
needs to be avoided. Raw Unicode characters within prover source files |
|
462 |
should be restricted to informal parts, e.g.\ to write text in non-latin |
|
463 |
alphabets in comments. |
|
57319 | 464 |
|
61415 | 465 |
\<^medskip> |
466 |
\paragraph{Encoding.} Technically, the Unicode view on Isabelle |
|
61477 | 467 |
symbols is an \<^emph>\<open>encoding\<close> called @{verbatim "UTF-8-Isabelle"} in jEdit |
60257 | 468 |
(not in the underlying JVM). It is provided by the Isabelle/jEdit plugin and |
469 |
enabled by default for all source files. Sometimes such defaults are reset |
|
470 |
accidentally, or malformed UTF-8 sequences in the text force jEdit to fall |
|
471 |
back on a different encoding like @{verbatim "ISO-8859-15"}. In that case, |
|
472 |
verbatim ``@{verbatim "\<alpha>"}'' will be shown in the text buffer instead of its |
|
61493 | 473 |
Unicode rendering ``\<open>\<alpha>\<close>''. The jEdit menu operation \<^emph>\<open>File~/ |
61477 | 474 |
Reload with Encoding~/ UTF-8-Isabelle\<close> helps to resolve such problems (after |
60257 | 475 |
repairing malformed parts of the text). |
57319 | 476 |
|
61415 | 477 |
\<^medskip> |
478 |
\paragraph{Font.} Correct rendering via Unicode requires a |
|
57319 | 479 |
font that contains glyphs for the corresponding codepoints. Most |
480 |
system fonts lack that, so Isabelle/jEdit prefers its own |
|
481 |
application font @{verbatim IsabelleText}, which ensures that |
|
482 |
standard collection of Isabelle symbols are actually seen on the |
|
483 |
screen (or printer). |
|
484 |
||
57420 | 485 |
Note that a Java/AWT/Swing application can load additional fonts only if |
486 |
they are not installed on the operating system already! Some outdated |
|
487 |
version of @{verbatim IsabelleText} that happens to be provided by the |
|
488 |
operating system would prevent Isabelle/jEdit to use its bundled version. |
|
489 |
This could lead to missing glyphs (black rectangles), when the system |
|
490 |
version of @{verbatim IsabelleText} is older than the application version. |
|
491 |
This problem can be avoided by refraining to ``install'' any version of |
|
492 |
@{verbatim IsabelleText} in the first place, although it is occasionally |
|
493 |
tempting to use the same font in other applications. |
|
57319 | 494 |
|
61415 | 495 |
\<^medskip> |
496 |
\paragraph{Input methods.} In principle, Isabelle/jEdit |
|
57319 | 497 |
could delegate the problem to produce Isabelle symbols in their |
498 |
Unicode rendering to the underlying operating system and its |
|
61477 | 499 |
\<^emph>\<open>input methods\<close>. Regular jEdit also provides various ways to |
500 |
work with \<^emph>\<open>abbreviations\<close> to produce certain non-ASCII |
|
57319 | 501 |
characters. Since none of these standard input methods work |
502 |
satisfactorily for the mathematical characters required for |
|
503 |
Isabelle, various specific Isabelle/jEdit mechanisms are provided. |
|
504 |
||
57420 | 505 |
This is a summary for practically relevant input methods for Isabelle |
506 |
symbols. |
|
57319 | 507 |
|
61477 | 508 |
\<^enum> The \<^emph>\<open>Symbols\<close> panel: some GUI buttons allow to insert |
57319 | 509 |
certain symbols in the text buffer. There are also tooltips to |
510 |
reveal the official Isabelle representation with some additional |
|
61477 | 511 |
information about \<^emph>\<open>symbol abbreviations\<close> (see below). |
57319 | 512 |
|
61415 | 513 |
\<^enum> Copy/paste from decoded source files: text that is rendered |
57319 | 514 |
as Unicode already can be re-used to produce further text. This |
515 |
also works between different applications, e.g.\ Isabelle/jEdit and |
|
516 |
some web browser or mail client, as long as the same Unicode view on |
|
517 |
Isabelle symbols is used. |
|
518 |
||
61415 | 519 |
\<^enum> Copy/paste from prover output within Isabelle/jEdit. The same |
61477 | 520 |
principles as for text buffers apply, but note that \<^emph>\<open>copy\<close> in secondary |
60257 | 521 |
Isabelle/jEdit windows works via the keyboard shortcuts @{verbatim "C+c"} or |
522 |
@{verbatim "C+INSERT"}, while jEdit menu actions always refer to the primary |
|
523 |
text area! |
|
57319 | 524 |
|
61415 | 525 |
\<^enum> Completion provided by Isabelle plugin (see |
57319 | 526 |
\secref{sec:completion}). Isabelle symbols have a canonical name |
527 |
and optional abbreviations. This can be used with the text |
|
528 |
completion mechanism of Isabelle/jEdit, to replace a prefix of the |
|
57328 | 529 |
actual symbol like @{verbatim "\<lambda>"}, or its name preceded by backslash |
57319 | 530 |
@{verbatim "\\"}@{verbatim "lambda"}, or its ASCII abbreviation |
531 |
@{verbatim "%"} by the Unicode rendering. |
|
532 |
||
533 |
The following table is an extract of the information provided by the |
|
534 |
standard @{file "$ISABELLE_HOME/etc/symbols"} file: |
|
535 |
||
61415 | 536 |
\<^medskip> |
57319 | 537 |
\begin{tabular}{lll} |
61477 | 538 |
\<^bold>\<open>symbol\<close> & \<^bold>\<open>name with backslash\<close> & \<^bold>\<open>abbreviation\<close> \\\hline |
61493 | 539 |
\<open>\<lambda>\<close> & @{verbatim "\\lambda"} & @{verbatim "%"} \\ |
540 |
\<open>\<Rightarrow>\<close> & @{verbatim "\\Rightarrow"} & @{verbatim "=>"} \\ |
|
541 |
\<open>\<Longrightarrow>\<close> & @{verbatim "\\Longrightarrow"} & @{verbatim "==>"} \\[0.5ex] |
|
542 |
\<open>\<And>\<close> & @{verbatim "\\And"} & @{verbatim "!!"} \\ |
|
543 |
\<open>\<equiv>\<close> & @{verbatim "\\equiv"} & @{verbatim "=="} \\[0.5ex] |
|
544 |
\<open>\<forall>\<close> & @{verbatim "\\forall"} & @{verbatim "!"} \\ |
|
545 |
\<open>\<exists>\<close> & @{verbatim "\\exists"} & @{verbatim "?"} \\ |
|
546 |
\<open>\<longrightarrow>\<close> & @{verbatim "\\longrightarrow"} & @{verbatim "-->"} \\ |
|
547 |
\<open>\<and>\<close> & @{verbatim "\\and"} & @{verbatim "&"} \\ |
|
548 |
\<open>\<or>\<close> & @{verbatim "\\or"} & @{verbatim "|"} \\ |
|
549 |
\<open>\<not>\<close> & @{verbatim "\\not"} & @{verbatim "~"} \\ |
|
550 |
\<open>\<noteq>\<close> & @{verbatim "\\noteq"} & @{verbatim "~="} \\ |
|
551 |
\<open>\<in>\<close> & @{verbatim "\\in"} & @{verbatim ":"} \\ |
|
552 |
\<open>\<notin>\<close> & @{verbatim "\\notin"} & @{verbatim "~:"} \\ |
|
57319 | 553 |
\end{tabular} |
61415 | 554 |
\<^medskip> |
555 |
||
57420 | 556 |
Note that the above abbreviations refer to the input method. The logical |
557 |
notation provides ASCII alternatives that often coincide, but sometimes |
|
558 |
deviate. This occasionally causes user confusion with very old-fashioned |
|
559 |
Isabelle source that use ASCII replacement notation like @{verbatim "!"} or |
|
560 |
@{verbatim "ALL"} directly in the text. |
|
57319 | 561 |
|
562 |
On the other hand, coincidence of symbol abbreviations with ASCII |
|
563 |
replacement syntax syntax helps to update old theory sources via |
|
564 |
explicit completion (see also @{verbatim "C+b"} explained in |
|
565 |
\secref{sec:completion}). |
|
566 |
||
567 |
||
568 |
\paragraph{Control symbols.} There are some special control symbols |
|
569 |
to modify the display style of a single symbol (without |
|
570 |
nesting). Control symbols may be applied to a region of selected |
|
61477 | 571 |
text, either using the \<^emph>\<open>Symbols\<close> panel or keyboard shortcuts or |
57319 | 572 |
jEdit actions. These editor operations produce a separate control |
573 |
symbol for each symbol in the text, in order to make the whole text |
|
574 |
appear in a certain style. |
|
575 |
||
61415 | 576 |
\<^medskip> |
57319 | 577 |
\begin{tabular}{llll} |
61477 | 578 |
\<^bold>\<open>style\<close> & \<^bold>\<open>symbol\<close> & \<^bold>\<open>shortcut\<close> & \<^bold>\<open>action\<close> \\\hline |
57329 | 579 |
superscript & @{verbatim "\<^sup>"} & @{verbatim "C+e UP"} & @{action_ref "isabelle.control-sup"} \\ |
580 |
subscript & @{verbatim "\<^sub>"} & @{verbatim "C+e DOWN"} & @{action_ref "isabelle.control-sub"} \\ |
|
581 |
bold face & @{verbatim "\<^bold>"} & @{verbatim "C+e RIGHT"} & @{action_ref "isabelle.control-bold"} \\ |
|
61483 | 582 |
emphasized & @{verbatim "\<^emph>"} & @{verbatim "C+e LEF"} & @{action_ref "isabelle.control-emph"} \\ |
583 |
reset & & @{verbatim "C+e BACK_SPACE"} & @{action_ref "isabelle.control-reset"} \\ |
|
57319 | 584 |
\end{tabular} |
61415 | 585 |
\<^medskip> |
61483 | 586 |
|
587 |
To produce a single control symbol, it is also possible to complete on |
|
588 |
@{verbatim "\\"}@{verbatim sup}, @{verbatim "\\"}@{verbatim sub}, @{verbatim |
|
589 |
"\\"}@{verbatim bold}, @{verbatim "\\"}@{verbatim emph} as for regular |
|
590 |
symbols. |
|
591 |
||
592 |
The emphasized style only takes effect in document output, not in the |
|
593 |
editor. |
|
594 |
\<close> |
|
57319 | 595 |
|
596 |
||
58618 | 597 |
section \<open>SideKick parsers \label{sec:sidekick}\<close> |
57319 | 598 |
|
58618 | 599 |
text \<open> |
61477 | 600 |
The \<^emph>\<open>SideKick\<close> plugin provides some general services to display buffer |
57319 | 601 |
structure in a tree view. |
602 |
||
57336 | 603 |
Isabelle/jEdit provides SideKick parsers for its main mode for theory files, |
604 |
as well as some minor modes for the @{verbatim NEWS} file (see |
|
605 |
\figref{fig:sidekick}), session @{verbatim ROOT} files, and system |
|
606 |
@{verbatim options}. |
|
607 |
||
608 |
\begin{figure}[htb] |
|
609 |
\begin{center} |
|
610 |
\includegraphics[scale=0.333]{sidekick} |
|
611 |
\end{center} |
|
612 |
\caption{The Isabelle NEWS file with SideKick tree view} |
|
613 |
\label{fig:sidekick} |
|
614 |
\end{figure} |
|
57319 | 615 |
|
616 |
Moreover, the special SideKick parser @{verbatim "isabelle-markup"} |
|
617 |
provides access to the full (uninterpreted) markup tree of the PIDE |
|
618 |
document model of the current buffer. This is occasionally useful |
|
619 |
for informative purposes, but the amount of displayed information |
|
620 |
might cause problems for large buffers, both for the human and the |
|
621 |
machine. |
|
58618 | 622 |
\<close> |
57319 | 623 |
|
624 |
||
58618 | 625 |
section \<open>Scala console \label{sec:scala-console}\<close> |
57319 | 626 |
|
58618 | 627 |
text \<open> |
61477 | 628 |
The \<^emph>\<open>Console\<close> plugin manages various shells (command interpreters), |
629 |
e.g.\ \<^emph>\<open>BeanShell\<close>, which is the official jEdit scripting language, and |
|
630 |
the cross-platform \<^emph>\<open>System\<close> shell. Thus the console provides similar |
|
57603 | 631 |
functionality than the Emacs buffers @{verbatim "*scratch*"} and |
57319 | 632 |
@{verbatim "*shell*"}. |
633 |
||
61477 | 634 |
Isabelle/jEdit extends the repertoire of the console by \<^emph>\<open>Scala\<close>, which |
57420 | 635 |
is the regular Scala toplevel loop running inside the same JVM process as |
636 |
Isabelle/jEdit itself. This means the Scala command interpreter has access |
|
57603 | 637 |
to the JVM name space and state of the running Prover IDE application. The |
638 |
default environment imports the full content of packages @{verbatim |
|
639 |
"isabelle"} and @{verbatim "isabelle.jedit"}. |
|
640 |
||
641 |
For example, @{verbatim PIDE} refers to the Isabelle/jEdit plugin object, |
|
642 |
and @{verbatim view} to the current editor view of jEdit. The Scala |
|
643 |
expression @{verbatim "PIDE.snapshot(view)"} makes a PIDE document snapshot |
|
644 |
of the current buffer within the current editor view. |
|
57319 | 645 |
|
646 |
This helps to explore Isabelle/Scala functionality interactively. Some care |
|
647 |
is required to avoid interference with the internals of the running |
|
648 |
application, especially in production use. |
|
58618 | 649 |
\<close> |
57319 | 650 |
|
651 |
||
58618 | 652 |
section \<open>File-system access\<close> |
57318 | 653 |
|
58618 | 654 |
text \<open> |
57420 | 655 |
File specifications in jEdit follow various formats and conventions |
61477 | 656 |
according to \<^emph>\<open>Virtual File Systems\<close>, which may be also provided by |
57420 | 657 |
additional plugins. This allows to access remote files via the @{verbatim |
658 |
"http:"} protocol prefix, for example. Isabelle/jEdit attempts to work with |
|
659 |
the file-system model of jEdit as far as possible. In particular, theory |
|
660 |
sources are passed directly from the editor to the prover, without |
|
661 |
indirection via physical files. |
|
57318 | 662 |
|
57420 | 663 |
Despite the flexibility of URLs in jEdit, local files are particularly |
664 |
important and are accessible without protocol prefix. Here the path notation |
|
665 |
is that of the Java Virtual Machine on the underlying platform. On Windows |
|
60257 | 666 |
the preferred form uses backslashes, but happens to accept also forward |
667 |
slashes like Unix/POSIX. Further differences arise due to Windows drive |
|
668 |
letters and network shares. |
|
57318 | 669 |
|
57331 | 670 |
The Java notation for files needs to be distinguished from the one of |
61477 | 671 |
Isabelle, which uses POSIX notation with forward slashes on \<^emph>\<open>all\<close> |
57331 | 672 |
platforms.\footnote{Isabelle/ML on Windows uses Cygwin file-system access |
673 |
and Unix-style path notation.} Moreover, environment variables from the |
|
57318 | 674 |
Isabelle process may be used freely, e.g.\ @{file |
675 |
"$ISABELLE_HOME/etc/symbols"} or @{file_unchecked "$POLYML_HOME/README"}. |
|
57331 | 676 |
There are special shortcuts: @{file "~"} for @{file "$USER_HOME"} and @{file |
677 |
"~~"} for @{file "$ISABELLE_HOME"}. |
|
57318 | 678 |
|
61415 | 679 |
\<^medskip> |
680 |
Since jEdit happens to support environment variables within file |
|
57420 | 681 |
specifications as well, it is natural to use similar notation within the |
682 |
editor, e.g.\ in the file-browser. This does not work in full generality, |
|
683 |
though, due to the bias of jEdit towards platform-specific notation and of |
|
684 |
Isabelle towards POSIX. Moreover, the Isabelle settings environment is not |
|
685 |
yet active when starting Isabelle/jEdit via its standard application |
|
60257 | 686 |
wrapper, in contrast to @{tool jedit} run from the command line |
687 |
(\secref{sec:command-line}). |
|
57318 | 688 |
|
57331 | 689 |
Isabelle/jEdit imitates @{verbatim "$ISABELLE_HOME"} and @{verbatim |
690 |
"$ISABELLE_HOME_USER"} within the Java process environment, in order to |
|
691 |
allow easy access to these important places from the editor. The file |
|
61477 | 692 |
browser of jEdit also includes \<^emph>\<open>Favorites\<close> for these two important |
57326 | 693 |
locations. |
57318 | 694 |
|
61415 | 695 |
\<^medskip> |
696 |
Path specifications in prover input or output usually include |
|
57318 | 697 |
formal markup that turns it into a hyperlink (see also |
698 |
\secref{sec:tooltips-hyperlinks}). This allows to open the corresponding |
|
699 |
file in the text editor, independently of the path notation. |
|
700 |
||
701 |
Formally checked paths in prover input are subject to completion |
|
57420 | 702 |
(\secref{sec:completion}): partial specifications are resolved via |
57318 | 703 |
directory content and possible completions are offered in a popup. |
58618 | 704 |
\<close> |
57318 | 705 |
|
706 |
||
58618 | 707 |
chapter \<open>Prover IDE functionality \label{sec:document-model}\<close> |
57315 | 708 |
|
58618 | 709 |
section \<open>Document model \label{sec:document-model}\<close> |
57322 | 710 |
|
58618 | 711 |
text \<open> |
57322 | 712 |
The document model is central to the PIDE architecture: the editor and the |
713 |
prover have a common notion of structured source text with markup, which is |
|
714 |
produced by formal processing. The editor is responsible for edits of |
|
715 |
document source, as produced by the user. The prover is responsible for |
|
716 |
reports of document markup, as produced by its processing in the background. |
|
717 |
||
718 |
Isabelle/jEdit handles classic editor events of jEdit, in order to connect |
|
719 |
the physical world of the GUI (with its singleton state) to the mathematical |
|
720 |
world of multiple document versions (with timeless and stateless updates). |
|
58618 | 721 |
\<close> |
57322 | 722 |
|
54322 | 723 |
|
58618 | 724 |
subsection \<open>Editor buffers and document nodes \label{sec:buffer-node}\<close> |
57322 | 725 |
|
58618 | 726 |
text \<open> |
61477 | 727 |
As a regular text editor, jEdit maintains a collection of \<^emph>\<open>buffers\<close> to |
57322 | 728 |
store text files; each buffer may be associated with any number of visible |
61477 | 729 |
\<^emph>\<open>text areas\<close>. Buffers are subject to an \<^emph>\<open>edit mode\<close> that is |
57322 | 730 |
determined from the file name extension. The following modes are treated |
731 |
specifically in Isabelle/jEdit: |
|
732 |
||
61415 | 733 |
\<^medskip> |
57322 | 734 |
\begin{tabular}{lll} |
61477 | 735 |
\<^bold>\<open>mode\<close> & \<^bold>\<open>file extension\<close> & \<^bold>\<open>content\<close> \\\hline |
57322 | 736 |
@{verbatim "isabelle"} & @{verbatim ".thy"} & theory source \\ |
737 |
@{verbatim "isabelle-ml"} & @{verbatim ".ML"} & Isabelle/ML source \\ |
|
738 |
@{verbatim "sml"} & @{verbatim ".sml"} or @{verbatim ".sig"} & Standard ML source \\ |
|
739 |
\end{tabular} |
|
61415 | 740 |
\<^medskip> |
54321 | 741 |
|
57322 | 742 |
All jEdit buffers are automatically added to the PIDE document-model as |
61477 | 743 |
\<^emph>\<open>document nodes\<close>. The overall document structure is defined by the |
57322 | 744 |
theory nodes in two dimensions: |
745 |
||
61477 | 746 |
\<^enum> via \<^bold>\<open>theory imports\<close> that are specified in the \<^emph>\<open>theory |
747 |
header\<close> using concrete syntax of the @{command_ref theory} command |
|
58554 | 748 |
@{cite "isabelle-isar-ref"}; |
57322 | 749 |
|
61477 | 750 |
\<^enum> via \<^bold>\<open>auxiliary files\<close> that are loaded into a theory by special |
751 |
\<^emph>\<open>load commands\<close>, notably @{command_ref ML_file} and @{command_ref |
|
58554 | 752 |
SML_file} @{cite "isabelle-isar-ref"}. |
57322 | 753 |
|
54322 | 754 |
|
57322 | 755 |
In any case, source files are managed by the PIDE infrastructure: the |
756 |
physical file-system only plays a subordinate role. The relevant version of |
|
60257 | 757 |
source text is passed directly from the editor to the prover, using internal |
57322 | 758 |
communication channels. |
58618 | 759 |
\<close> |
57322 | 760 |
|
761 |
||
58618 | 762 |
subsection \<open>Theories \label{sec:theories}\<close> |
57322 | 763 |
|
58618 | 764 |
text \<open> |
61477 | 765 |
The \<^emph>\<open>Theories\<close> panel (see also \figref{fig:theories}) provides an |
57322 | 766 |
overview of the status of continuous checking of theory nodes within the |
58554 | 767 |
document model. Unlike batch sessions of @{tool build} @{cite |
60270 | 768 |
"isabelle-system"}, theory nodes are identified by full path names; this allows |
58554 | 769 |
to work with multiple (disjoint) Isabelle sessions simultaneously within the |
770 |
same editor session. |
|
57322 | 771 |
|
57339 | 772 |
\begin{figure}[htb] |
773 |
\begin{center} |
|
774 |
\includegraphics[scale=0.333]{theories} |
|
775 |
\end{center} |
|
776 |
\caption{Theories panel with an overview of the document-model, and some |
|
777 |
jEdit text areas as editable view on some of the document nodes} |
|
778 |
\label{fig:theories} |
|
779 |
\end{figure} |
|
780 |
||
57322 | 781 |
Certain events to open or update editor buffers cause Isabelle/jEdit to |
782 |
resolve dependencies of theory imports. The system requests to load |
|
783 |
additional files into editor buffers, in order to be included in the |
|
784 |
document model for further checking. It is also possible to let the system |
|
57420 | 785 |
resolve dependencies automatically, according to the system option |
786 |
@{system_option jedit_auto_load}. |
|
54321 | 787 |
|
61415 | 788 |
\<^medskip> |
61477 | 789 |
The visible \<^emph>\<open>perspective\<close> of Isabelle/jEdit is defined by the |
57322 | 790 |
collective view on theory buffers via open text areas. The perspective is |
791 |
taken as a hint for document processing: the prover ensures that those parts |
|
792 |
of a theory where the user is looking are checked, while other parts that |
|
793 |
are presently not required are ignored. The perspective is changed by |
|
794 |
opening or closing text area windows, or scrolling within a window. |
|
54322 | 795 |
|
61477 | 796 |
The \<^emph>\<open>Theories\<close> panel provides some further options to influence |
54330 | 797 |
the process of continuous checking: it may be switched off globally |
54350 | 798 |
to restrict the prover to superficial processing of command syntax. |
61477 | 799 |
It is also possible to indicate theory nodes as \<^emph>\<open>required\<close> for |
54330 | 800 |
continuous checking: this means such nodes and all their imports are |
801 |
always processed independently of the visibility status (if |
|
802 |
continuous checking is enabled). Big theory libraries that are |
|
803 |
marked as required can have significant impact on performance, |
|
804 |
though. |
|
54322 | 805 |
|
61415 | 806 |
\<^medskip> |
807 |
Formal markup of checked theory content is turned into GUI |
|
57310 | 808 |
rendering, based on a standard repertoire known from IDEs for programming |
57420 | 809 |
languages: colors, icons, highlighting, squiggly underlines, tooltips, |
57310 | 810 |
hyperlinks etc. For outer syntax of Isabelle/Isar there is some traditional |
60257 | 811 |
syntax-highlighting via static keywords and tokenization within the editor; |
812 |
this buffer syntax is determined from theory imports. In contrast, the |
|
813 |
painting of inner syntax (term language etc.)\ uses semantic information |
|
814 |
that is reported dynamically from the logical context. Thus the prover can |
|
815 |
provide additional markup to help the user to understand the meaning of |
|
816 |
formal text, and to produce more text with some add-on tools (e.g.\ |
|
61477 | 817 |
information messages with \<^emph>\<open>sendback\<close> markup by automated provers or |
60257 | 818 |
disprovers in the background). |
57322 | 819 |
|
58618 | 820 |
\<close> |
57322 | 821 |
|
58618 | 822 |
subsection \<open>Auxiliary files \label{sec:aux-files}\<close> |
57322 | 823 |
|
58618 | 824 |
text \<open> |
57329 | 825 |
Special load commands like @{command_ref ML_file} and @{command_ref |
58554 | 826 |
SML_file} @{cite "isabelle-isar-ref"} refer to auxiliary files within some |
57329 | 827 |
theory. Conceptually, the file argument of the command extends the theory |
828 |
source by the content of the file, but its editor buffer may be loaded~/ |
|
829 |
changed~/ saved separately. The PIDE document model propagates changes of |
|
830 |
auxiliary file content to the corresponding load command in the theory, to |
|
831 |
update and process it accordingly: changes of auxiliary file content are |
|
832 |
treated as changes of the corresponding load command. |
|
57323 | 833 |
|
61415 | 834 |
\<^medskip> |
835 |
As a concession to the massive amount of ML files in Isabelle/HOL |
|
57323 | 836 |
itself, the content of auxiliary files is only added to the PIDE |
837 |
document-model on demand, the first time when opened explicitly in the |
|
57420 | 838 |
editor. There are further tricks to manage markup of ML files, such that |
839 |
Isabelle/HOL may be edited conveniently in the Prover IDE on small machines |
|
60257 | 840 |
with only 8\,GB of main memory. Using @{verbatim Pure} as logic session |
57420 | 841 |
image, the exploration may start at the top @{file |
57323 | 842 |
"$ISABELLE_HOME/src/HOL/Main.thy"} or the bottom @{file |
843 |
"$ISABELLE_HOME/src/HOL/HOL.thy"}, for example. |
|
844 |
||
845 |
Initially, before an auxiliary file is opened in the editor, the prover |
|
846 |
reads its content from the physical file-system. After the file is opened |
|
847 |
for the first time in the editor, e.g.\ by following the hyperlink |
|
848 |
(\secref{sec:tooltips-hyperlinks}) for the argument of its @{command |
|
849 |
ML_file} command, the content is taken from the jEdit buffer. |
|
850 |
||
851 |
The change of responsibility from prover to editor counts as an update of |
|
852 |
the document content, so subsequent theory sources need to be re-checked. |
|
57420 | 853 |
When the buffer is closed, the responsibility remains to the editor: the |
854 |
file may be opened again without causing another document update. |
|
57323 | 855 |
|
856 |
A file that is opened in the editor, but its theory with the load command is |
|
857 |
not, is presently inactive in the document model. A file that is loaded via |
|
858 |
multiple load commands is associated to an arbitrary one: this situation is |
|
859 |
morally unsupported and might lead to confusion. |
|
860 |
||
61415 | 861 |
\<^medskip> |
862 |
Output that refers to an auxiliary file is combined with that of |
|
57323 | 863 |
the corresponding load command, and shown whenever the file or the command |
864 |
are active (see also \secref{sec:output}). |
|
865 |
||
866 |
Warnings, errors, and other useful markup is attached directly to the |
|
867 |
positions in the auxiliary file buffer, in the manner of other well-known |
|
868 |
IDEs. By using the load command @{command SML_file} as explained in @{file |
|
869 |
"$ISABELLE_HOME/src/Tools/SML/Examples.thy"}, Isabelle/jEdit may be used as |
|
870 |
fully-featured IDE for Standard ML, independently of theory or proof |
|
871 |
development: the required theory merely serves as some kind of project |
|
872 |
file for a collection of SML source modules. |
|
58618 | 873 |
\<close> |
54322 | 874 |
|
54352 | 875 |
|
58618 | 876 |
section \<open>Output \label{sec:output}\<close> |
54353 | 877 |
|
58618 | 878 |
text \<open> |
61477 | 879 |
Prover output consists of \<^emph>\<open>markup\<close> and \<^emph>\<open>messages\<close>. Both are |
57420 | 880 |
directly attached to the corresponding positions in the original source |
881 |
text, and visualized in the text area, e.g.\ as text colours for free and |
|
882 |
bound variables, or as squiggly underlines for warnings, errors etc.\ (see |
|
883 |
also \figref{fig:output}). In the latter case, the corresponding messages |
|
884 |
are shown by hovering with the mouse over the highlighted text --- although |
|
885 |
in many situations the user should already get some clue by looking at the |
|
886 |
position of the text highlighting, without the text itself. |
|
54357 | 887 |
|
888 |
\begin{figure}[htb] |
|
889 |
\begin{center} |
|
57312 | 890 |
\includegraphics[scale=0.333]{output} |
54357 | 891 |
\end{center} |
54372 | 892 |
\caption{Multiple views on prover output: gutter area with icon, |
893 |
text area with popup, overview area, Theories panel, Output panel} |
|
54357 | 894 |
\label{fig:output} |
895 |
\end{figure} |
|
54353 | 896 |
|
897 |
The ``gutter area'' on the left-hand-side of the text area uses |
|
54372 | 898 |
icons to provide a summary of the messages within the adjacent |
54353 | 899 |
line of text. Message priorities are used to prefer errors over |
57310 | 900 |
warnings, warnings over information messages, but plain output is |
901 |
ignored. |
|
54353 | 902 |
|
57310 | 903 |
The ``overview area'' on the right-hand-side of the text area uses similar |
904 |
information to paint small rectangles for the overall status of the whole |
|
905 |
text buffer. The graphics is scaled to fit the logical buffer length into |
|
906 |
the given window height. Mouse clicks on the overview area position the |
|
907 |
cursor approximately to the corresponding line of text in the buffer. |
|
54353 | 908 |
|
61477 | 909 |
Another course-grained overview is provided by the \<^emph>\<open>Theories\<close> |
54372 | 910 |
panel, but without direct correspondence to text positions. A |
911 |
double-click on one of the theory entries with their status overview |
|
912 |
opens the corresponding text buffer, without changing the cursor |
|
913 |
position. |
|
54353 | 914 |
|
61415 | 915 |
\<^medskip> |
61477 | 916 |
In addition, the \<^emph>\<open>Output\<close> panel displays prover |
54353 | 917 |
messages that correspond to a given command, within a separate |
918 |
window. |
|
919 |
||
57310 | 920 |
The cursor position in the presently active text area determines the prover |
921 |
command whose cumulative message output is appended and shown in that window |
|
922 |
(in canonical order according to the internal execution of the command). |
|
923 |
There are also control elements to modify the update policy of the output |
|
924 |
wrt.\ continued editor movements. This is particularly useful with several |
|
61477 | 925 |
independent instances of the \<^emph>\<open>Output\<close> panel, which the Dockable Window |
57310 | 926 |
Manager of jEdit can handle conveniently. |
54353 | 927 |
|
57310 | 928 |
Former users of the old TTY interaction model (e.g.\ Proof~General) might |
929 |
find a separate window for prover messages familiar, but it is important to |
|
930 |
understand that the main Prover IDE feedback happens elsewhere. It is |
|
57420 | 931 |
possible to do meaningful proof editing within the primary text area and its |
932 |
markup, while using secondary output windows only rarely. |
|
54353 | 933 |
|
934 |
The main purpose of the output window is to ``debug'' unclear |
|
935 |
situations by inspecting internal state of the prover.\footnote{In |
|
54355 | 936 |
that sense, unstructured tactic scripts depend on continuous |
54353 | 937 |
debugging with internal state inspection.} Consequently, some |
61477 | 938 |
special messages for \<^emph>\<open>tracing\<close> or \<^emph>\<open>proof state\<close> only |
54353 | 939 |
appear here, and are not attached to the original source. |
940 |
||
61415 | 941 |
\<^medskip> |
942 |
In any case, prover messages also contain markup that may |
|
54353 | 943 |
be explored recursively via tooltips or hyperlinks (see |
944 |
\secref{sec:tooltips-hyperlinks}), or clicked directly to initiate |
|
54355 | 945 |
certain actions (see \secref{sec:auto-tools} and |
58618 | 946 |
\secref{sec:sledgehammer}).\<close> |
54353 | 947 |
|
948 |
||
58618 | 949 |
section \<open>Query \label{sec:query}\<close> |
57311 | 950 |
|
58618 | 951 |
text \<open> |
61477 | 952 |
The \<^emph>\<open>Query\<close> panel provides various GUI forms to request extra |
57420 | 953 |
information from the prover. In old times the user would have issued some |
57314 | 954 |
diagnostic command like @{command find_theorems} and inspected its output, |
955 |
but this is now integrated into the Prover IDE. |
|
57311 | 956 |
|
61477 | 957 |
A \<^emph>\<open>Query\<close> window provides some input fields and buttons for a |
57311 | 958 |
particular query command, with output in a dedicated text area. There are |
61477 | 959 |
various query modes: \<^emph>\<open>Find Theorems\<close>, \<^emph>\<open>Find Constants\<close>, |
960 |
\<^emph>\<open>Print Context\<close>, e.g.\ see \figref{fig:query}. As usual in jEdit, |
|
961 |
multiple \<^emph>\<open>Query\<close> windows may be active at the same time: any number of |
|
57313 | 962 |
floating instances, but at most one docked instance (which is used by |
963 |
default). |
|
964 |
||
965 |
\begin{figure}[htb] |
|
966 |
\begin{center} |
|
967 |
\includegraphics[scale=0.333]{query} |
|
968 |
\end{center} |
|
969 |
\caption{An instance of the Query panel} |
|
970 |
\label{fig:query} |
|
971 |
\end{figure} |
|
57311 | 972 |
|
61415 | 973 |
\<^medskip> |
974 |
The following GUI elements are common to all query modes: |
|
57311 | 975 |
|
61415 | 976 |
\<^item> The spinning wheel provides feedback about the status of a pending |
57311 | 977 |
query wrt.\ the evaluation of its context and its own operation. |
978 |
||
61477 | 979 |
\<^item> The \<^emph>\<open>Apply\<close> button attaches a fresh query invocation to the |
57311 | 980 |
current context of the command where the cursor is pointing in the text. |
981 |
||
61477 | 982 |
\<^item> The \<^emph>\<open>Search\<close> field allows to highlight query output according to |
57313 | 983 |
some regular expression, in the notation that is commonly used on the Java |
57420 | 984 |
platform.\footnote{@{url |
985 |
"http://docs.oracle.com/javase/7/docs/api/java/util/regex/Pattern.html"}} |
|
986 |
This may serve as an additional visual filter of the result. |
|
57311 | 987 |
|
61477 | 988 |
\<^item> The \<^emph>\<open>Zoom\<close> box controls the font size of the output area. |
57311 | 989 |
|
990 |
||
991 |
All query operations are asynchronous: there is no need to wait for the |
|
992 |
evaluation of the document for the query context, nor for the query |
|
61477 | 993 |
operation itself. Query output may be detached as independent \<^emph>\<open>Info\<close> |
57311 | 994 |
window, using a menu operation of the dockable window manager. The printed |
995 |
result usually provides sufficient clues about the original query, with some |
|
996 |
hyperlink to its context (via markup of its head line). |
|
58618 | 997 |
\<close> |
57311 | 998 |
|
999 |
||
58618 | 1000 |
subsection \<open>Find theorems\<close> |
57311 | 1001 |
|
58618 | 1002 |
text \<open> |
61477 | 1003 |
The \<^emph>\<open>Query\<close> panel in \<^emph>\<open>Find Theorems\<close> mode retrieves facts from the |
1004 |
theory or proof context matching all of given criteria in the \<^emph>\<open>Find\<close> |
|
57313 | 1005 |
text field. A single criterium has the following syntax: |
57311 | 1006 |
|
57313 | 1007 |
@{rail \<open> |
1008 |
('-'?) ('name' ':' @{syntax nameref} | 'intro' | 'elim' | 'dest' | |
|
1009 |
'solves' | 'simp' ':' @{syntax term} | @{syntax term}) |
|
1010 |
\<close>} |
|
1011 |
||
57329 | 1012 |
See also the Isar command @{command_ref find_theorems} in |
58554 | 1013 |
@{cite "isabelle-isar-ref"}. |
58618 | 1014 |
\<close> |
57311 | 1015 |
|
1016 |
||
58618 | 1017 |
subsection \<open>Find constants\<close> |
57311 | 1018 |
|
58618 | 1019 |
text \<open> |
61477 | 1020 |
The \<^emph>\<open>Query\<close> panel in \<^emph>\<open>Find Constants\<close> mode prints all constants |
1021 |
whose type meets all of the given criteria in the \<^emph>\<open>Find\<close> text field. |
|
57313 | 1022 |
A single criterium has the following syntax: |
1023 |
||
1024 |
@{rail \<open> |
|
1025 |
('-'?) |
|
1026 |
('name' ':' @{syntax nameref} | 'strict' ':' @{syntax type} | @{syntax type}) |
|
1027 |
\<close>} |
|
1028 |
||
58554 | 1029 |
See also the Isar command @{command_ref find_consts} in @{cite |
1030 |
"isabelle-isar-ref"}. |
|
58618 | 1031 |
\<close> |
57311 | 1032 |
|
1033 |
||
58618 | 1034 |
subsection \<open>Print context\<close> |
57311 | 1035 |
|
58618 | 1036 |
text \<open> |
61477 | 1037 |
The \<^emph>\<open>Query\<close> panel in \<^emph>\<open>Print Context\<close> mode prints information from |
57313 | 1038 |
the theory or proof context, or proof state. See also the Isar commands |
57329 | 1039 |
@{command_ref print_context}, @{command_ref print_cases}, @{command_ref |
58554 | 1040 |
print_term_bindings}, @{command_ref print_theorems}, @{command_ref |
1041 |
print_state} described in @{cite "isabelle-isar-ref"}. |
|
58618 | 1042 |
\<close> |
57311 | 1043 |
|
1044 |
||
58618 | 1045 |
section \<open>Tooltips and hyperlinks \label{sec:tooltips-hyperlinks}\<close> |
54352 | 1046 |
|
58618 | 1047 |
text \<open> |
57310 | 1048 |
Formally processed text (prover input or output) contains rich markup |
1049 |
information that can be explored further by using the @{verbatim CONTROL} |
|
1050 |
modifier key on Linux and Windows, or @{verbatim COMMAND} on Mac OS X. |
|
1051 |
Hovering with the mouse while the modifier is pressed reveals a |
|
61477 | 1052 |
\<^emph>\<open>tooltip\<close> (grey box over the text with a yellow popup) and/or a |
1053 |
\<^emph>\<open>hyperlink\<close> (black rectangle over the text with change of mouse |
|
57310 | 1054 |
pointer); see also \figref{fig:tooltip}. |
54331 | 1055 |
|
54357 | 1056 |
\begin{figure}[htb] |
54331 | 1057 |
\begin{center} |
57312 | 1058 |
\includegraphics[scale=0.5]{popup1} |
54331 | 1059 |
\end{center} |
54356 | 1060 |
\caption{Tooltip and hyperlink for some formal entity} |
54350 | 1061 |
\label{fig:tooltip} |
54331 | 1062 |
\end{figure} |
1063 |
||
57310 | 1064 |
Tooltip popups use the same rendering mechanisms as the main text |
54350 | 1065 |
area, and further tooltips and/or hyperlinks may be exposed |
54357 | 1066 |
recursively by the same mechanism; see \figref{fig:nested-tooltips}. |
54323 | 1067 |
|
54357 | 1068 |
\begin{figure}[htb] |
54331 | 1069 |
\begin{center} |
57312 | 1070 |
\includegraphics[scale=0.5]{popup2} |
54331 | 1071 |
\end{center} |
54356 | 1072 |
\caption{Nested tooltips over formal entities} |
54350 | 1073 |
\label{fig:nested-tooltips} |
54331 | 1074 |
\end{figure} |
54350 | 1075 |
|
61477 | 1076 |
The tooltip popup window provides some controls to \<^emph>\<open>close\<close> or |
1077 |
\<^emph>\<open>detach\<close> the window, turning it into a separate \<^emph>\<open>Info\<close> |
|
54372 | 1078 |
window managed by jEdit. The @{verbatim ESCAPE} key closes |
61477 | 1079 |
\<^emph>\<open>all\<close> popups, which is particularly relevant when nested |
54352 | 1080 |
tooltips are stacking up. |
1081 |
||
61415 | 1082 |
\<^medskip> |
1083 |
A black rectangle in the text indicates a hyperlink that may be |
|
57310 | 1084 |
followed by a mouse click (while the @{verbatim CONTROL} or @{verbatim |
1085 |
COMMAND} modifier key is still pressed). Such jumps to other text locations |
|
61477 | 1086 |
are recorded by the \<^emph>\<open>Navigator\<close> plugin, which is bundled with |
57310 | 1087 |
Isabelle/jEdit and enabled by default, including navigation arrows in the |
1088 |
main jEdit toolbar. |
|
54352 | 1089 |
|
1090 |
Also note that the link target may be a file that is itself not |
|
1091 |
subject to formal document processing of the editor session and thus |
|
1092 |
prevents further exploration: the chain of hyperlinks may end in |
|
54372 | 1093 |
some source file of the underlying logic image, or within the |
60257 | 1094 |
ML bootstrap sources of Isabelle/Pure.\<close> |
54321 | 1095 |
|
1096 |
||
58618 | 1097 |
section \<open>Completion \label{sec:completion}\<close> |
57324 | 1098 |
|
58618 | 1099 |
text \<open> |
61477 | 1100 |
Smart completion of partial input is the IDE functionality \<^emph>\<open>par |
1101 |
excellance\<close>. Isabelle/jEdit combines several sources of information to |
|
57328 | 1102 |
achieve that. Despite its complexity, it should be possible to get some idea |
1103 |
how completion works by experimentation, based on the overview of completion |
|
57335 | 1104 |
varieties in \secref{sec:completion-varieties}. The remaining subsections |
1105 |
explain concepts around completion more systematically. |
|
57325 | 1106 |
|
61415 | 1107 |
\<^medskip> |
61477 | 1108 |
\<^emph>\<open>Explicit completion\<close> is triggered by the action @{action_ref |
57335 | 1109 |
"isabelle.complete"}, which is bound to the keyboard shortcut @{verbatim |
1110 |
"C+b"}, and thus overrides the jEdit default for @{action_ref |
|
1111 |
"complete-word"}. |
|
1112 |
||
61477 | 1113 |
\<^emph>\<open>Implicit completion\<close> hooks into the regular keyboard input stream of |
57335 | 1114 |
the editor, with some event filtering and optional delays. |
54361 | 1115 |
|
61415 | 1116 |
\<^medskip> |
61477 | 1117 |
Completion options may be configured in \<^emph>\<open>Plugin Options~/ |
1118 |
Isabelle~/ General~/ Completion\<close>. These are explained in further detail |
|
57328 | 1119 |
below, whenever relevant. There is also a summary of options in |
1120 |
\secref{sec:completion-options}. |
|
1121 |
||
57335 | 1122 |
The asynchronous nature of PIDE interaction means that information from the |
1123 |
prover is delayed --- at least by a full round-trip of the document update |
|
1124 |
protocol. The default options already take this into account, with a |
|
57324 | 1125 |
sufficiently long completion delay to speculate on the availability of all |
57335 | 1126 |
relevant information from the editor and the prover, before completing text |
1127 |
immediately or producing a popup. Although there is an inherent danger of |
|
1128 |
non-deterministic behaviour due to such real-time parameters, the general |
|
1129 |
completion policy aims at determined results as far as possible. |
|
58618 | 1130 |
\<close> |
57324 | 1131 |
|
1132 |
||
58618 | 1133 |
subsection \<open>Varieties of completion \label{sec:completion-varieties}\<close> |
57324 | 1134 |
|
58618 | 1135 |
subsubsection \<open>Built-in templates\<close> |
57324 | 1136 |
|
58618 | 1137 |
text \<open> |
57327 | 1138 |
Isabelle is ultimately a framework of nested sub-languages of different |
57328 | 1139 |
kinds and purposes. The completion mechanism supports this by the following |
1140 |
built-in templates: |
|
1141 |
||
61477 | 1142 |
\<^descr> @{verbatim "`"} (single ASCII back-quote) supports \<^emph>\<open>quotations\<close> |
57327 | 1143 |
via text cartouches. There are three selections, which are always presented |
57328 | 1144 |
in the same order and do not depend on any context information. The default |
61493 | 1145 |
choice produces a template ``\<open>\<open>\<box>\<close>\<close>'', where the box indicates the |
57327 | 1146 |
cursor position after insertion; the other choices help to repair the block |
1147 |
structure of unbalanced text cartouches. |
|
57324 | 1148 |
|
61493 | 1149 |
\<^descr> @{verbatim "@{"} is completed to the template ``\<open>@{\<box>}\<close>'', |
57335 | 1150 |
where the box indicates the cursor position after insertion. Here it is |
1151 |
convenient to use the wildcard ``@{verbatim __}'' or a more specific name |
|
1152 |
prefix to let semantic completion of name-space entries propose |
|
1153 |
antiquotation names. |
|
1154 |
||
1155 |
||
1156 |
With some practice, input of quoted sub-languages and antiquotations of |
|
1157 |
embedded languages should work fluently. Note that national keyboard layouts |
|
1158 |
might cause problems with back-quote as dead key: if possible, dead keys |
|
1159 |
should be disabled. |
|
58618 | 1160 |
\<close> |
57335 | 1161 |
|
57327 | 1162 |
|
58618 | 1163 |
subsubsection \<open>Syntax keywords\<close> |
57335 | 1164 |
|
58618 | 1165 |
text \<open> |
57335 | 1166 |
Syntax completion tables are determined statically from the keywords of the |
1167 |
``outer syntax'' of the underlying edit mode: for theory files this is the |
|
60257 | 1168 |
syntax of Isar commands according to the cumulative theory imports. |
57327 | 1169 |
|
57335 | 1170 |
Keywords are usually plain words, which means the completion mechanism only |
1171 |
inserts them directly into the text for explicit completion |
|
1172 |
(\secref{sec:completion-input}), but produces a popup |
|
1173 |
(\secref{sec:completion-popup}) otherwise. |
|
1174 |
||
1175 |
At the point where outer syntax keywords are defined, it is possible to |
|
1176 |
specify an alternative replacement string to be inserted instead of the |
|
1177 |
keyword itself. An empty string means to suppress the keyword altogether, |
|
1178 |
which is occasionally useful to avoid confusion, e.g.\ the rare keyword |
|
61493 | 1179 |
@{command simproc_setup} vs.\ the frequent name-space entry \<open>simp\<close>. |
58618 | 1180 |
\<close> |
57324 | 1181 |
|
1182 |
||
58618 | 1183 |
subsubsection \<open>Isabelle symbols\<close> |
57324 | 1184 |
|
58618 | 1185 |
text \<open> |
57325 | 1186 |
The completion tables for Isabelle symbols (\secref{sec:symbols}) are |
1187 |
determined statically from @{file "$ISABELLE_HOME/etc/symbols"} and |
|
57328 | 1188 |
@{file_unchecked "$ISABELLE_HOME_USER/etc/symbols"} for each symbol |
1189 |
specification as follows: |
|
57325 | 1190 |
|
61415 | 1191 |
\<^medskip> |
57325 | 1192 |
\begin{tabular}{ll} |
61477 | 1193 |
\<^bold>\<open>completion entry\<close> & \<^bold>\<open>example\<close> \\\hline |
57325 | 1194 |
literal symbol & @{verbatim "\<forall>"} \\ |
57328 | 1195 |
symbol name with backslash & @{verbatim "\\"}@{verbatim forall} \\ |
57335 | 1196 |
symbol abbreviation & @{verbatim "ALL"} or @{verbatim "!"} \\ |
57325 | 1197 |
\end{tabular} |
61415 | 1198 |
\<^medskip> |
57325 | 1199 |
|
57335 | 1200 |
When inserted into the text, the above examples all produce the same Unicode |
61493 | 1201 |
rendering \<open>\<forall>\<close> of the underlying symbol @{verbatim "\<forall>"}. |
57325 | 1202 |
|
57335 | 1203 |
A symbol abbreviation that is a plain word, like @{verbatim "ALL"}, is |
1204 |
treated like a syntax keyword. Non-word abbreviations like @{verbatim "-->"} |
|
1205 |
are inserted more aggressively, except for single-character abbreviations |
|
1206 |
like @{verbatim "!"} above. |
|
57324 | 1207 |
|
61415 | 1208 |
\<^medskip> |
1209 |
Symbol completion depends on the semantic language context |
|
57335 | 1210 |
(\secref{sec:completion-context}), to enable or disable that aspect for a |
1211 |
particular sub-language of Isabelle. For example, symbol completion is |
|
1212 |
suppressed within document source to avoid confusion with {\LaTeX} macros |
|
1213 |
that use similar notation. |
|
58618 | 1214 |
\<close> |
57324 | 1215 |
|
1216 |
||
58618 | 1217 |
subsubsection \<open>Name-space entries\<close> |
57324 | 1218 |
|
58618 | 1219 |
text \<open> |
57324 | 1220 |
This is genuine semantic completion, using information from the prover, so |
61477 | 1221 |
it requires some delay. A \<^emph>\<open>failed name-space lookup\<close> produces an error |
57335 | 1222 |
message that is annotated with a list of alternative names that are legal. |
1223 |
The list of results is truncated according to the system option |
|
1224 |
@{system_option_ref completion_limit}. The completion mechanism takes this |
|
1225 |
into account when collecting information on the prover side. |
|
57324 | 1226 |
|
61477 | 1227 |
Already recognized names are \<^emph>\<open>not\<close> completed further, but completion |
57328 | 1228 |
may be extended by appending a suffix of underscores. This provokes a failed |
1229 |
lookup, and another completion attempt while ignoring the underscores. For |
|
1230 |
example, in a name space where @{verbatim "foo"} and @{verbatim "foobar"} |
|
1231 |
are known, the input @{verbatim "foo"} remains unchanged, but @{verbatim |
|
1232 |
"foo_"} may be completed to @{verbatim "foo"} or @{verbatim "foobar"}. |
|
57324 | 1233 |
|
57326 | 1234 |
The special identifier ``@{verbatim "__"}'' serves as a wild-card for |
1235 |
arbitrary completion: it exposes the name-space content to the completion |
|
1236 |
mechanism (truncated according to @{system_option completion_limit}). This |
|
1237 |
is occasionally useful to explore an unknown name-space, e.g.\ in some |
|
57324 | 1238 |
template. |
58618 | 1239 |
\<close> |
57324 | 1240 |
|
1241 |
||
58618 | 1242 |
subsubsection \<open>File-system paths\<close> |
57324 | 1243 |
|
58618 | 1244 |
text \<open> |
57324 | 1245 |
Depending on prover markup about file-system path specifications in the |
57335 | 1246 |
source text, e.g.\ for the argument of a load command |
57324 | 1247 |
(\secref{sec:aux-files}), the completion mechanism explores the directory |
1248 |
content and offers the result as completion popup. Relative path |
|
61477 | 1249 |
specifications are understood wrt.\ the \<^emph>\<open>master directory\<close> of the |
57335 | 1250 |
document node (\secref{sec:buffer-node}) of the enclosing editor buffer; |
1251 |
this requires a proper theory, not an auxiliary file. |
|
57324 | 1252 |
|
1253 |
A suffix of slashes may be used to continue the exploration of an already |
|
1254 |
recognized directory name. |
|
58618 | 1255 |
\<close> |
57324 | 1256 |
|
1257 |
||
58618 | 1258 |
subsubsection \<open>Spell-checking\<close> |
57328 | 1259 |
|
58618 | 1260 |
text \<open> |
57328 | 1261 |
The spell-checker combines semantic markup from the prover (regions of plain |
1262 |
words) with static dictionaries (word lists) that are known to the editor. |
|
1263 |
||
57333 | 1264 |
Unknown words are underlined in the text, using @{system_option_ref |
57328 | 1265 |
spell_checker_color} (blue by default). This is not an error, but a hint to |
57335 | 1266 |
the user that some action may be taken. The jEdit context menu provides |
1267 |
various actions, as far as applicable: |
|
57328 | 1268 |
|
61415 | 1269 |
\<^medskip> |
57328 | 1270 |
\begin{tabular}{l} |
57329 | 1271 |
@{action_ref "isabelle.complete-word"} \\ |
1272 |
@{action_ref "isabelle.exclude-word"} \\ |
|
1273 |
@{action_ref "isabelle.exclude-word-permanently"} \\ |
|
1274 |
@{action_ref "isabelle.include-word"} \\ |
|
1275 |
@{action_ref "isabelle.include-word-permanently"} \\ |
|
57328 | 1276 |
\end{tabular} |
61415 | 1277 |
\<^medskip> |
57328 | 1278 |
|
57329 | 1279 |
Instead of the specific @{action_ref "isabelle.complete-word"}, it is also |
1280 |
possible to use the generic @{action_ref "isabelle.complete"} with its |
|
57335 | 1281 |
default keyboard shortcut @{verbatim "C+b"}. |
57328 | 1282 |
|
61415 | 1283 |
\<^medskip> |
1284 |
Dictionary lookup uses some educated guesses about lower-case, |
|
57328 | 1285 |
upper-case, and capitalized words. This is oriented on common use in |
57335 | 1286 |
English, where this aspect is not decisive for proper spelling, in contrast |
1287 |
to German, for example. |
|
58618 | 1288 |
\<close> |
57328 | 1289 |
|
1290 |
||
58618 | 1291 |
subsection \<open>Semantic completion context \label{sec:completion-context}\<close> |
57325 | 1292 |
|
58618 | 1293 |
text \<open> |
57325 | 1294 |
Completion depends on a semantic context that is provided by the prover, |
1295 |
although with some delay, because at least a full PIDE protocol round-trip |
|
1296 |
is required. Until that information becomes available in the PIDE |
|
1297 |
document-model, the default context is given by the outer syntax of the |
|
1298 |
editor mode (see also \secref{sec:buffer-node}). |
|
1299 |
||
61477 | 1300 |
The semantic \<^emph>\<open>language context\<close> provides information about nested |
57335 | 1301 |
sub-languages of Isabelle: keywords are only completed for outer syntax, |
1302 |
symbols or antiquotations for languages that support them. E.g.\ there is no |
|
1303 |
symbol completion for ML source, but within ML strings, comments, |
|
1304 |
antiquotations. |
|
57325 | 1305 |
|
61477 | 1306 |
The prover may produce \<^emph>\<open>no completion\<close> markup in exceptional |
57335 | 1307 |
situations, to tell that some language keywords should be excluded from |
1308 |
further completion attempts. For example, @{verbatim ":"} within accepted |
|
61493 | 1309 |
Isar syntax looses its meaning as abbreviation for symbol \<open>\<in>\<close>. |
57589 | 1310 |
|
61415 | 1311 |
\<^medskip> |
61477 | 1312 |
The completion context is \<^emph>\<open>ignored\<close> for built-in templates and |
57589 | 1313 |
symbols in their explicit form ``@{verbatim "\<foobar>"}''; see also |
1314 |
\secref{sec:completion-varieties}. This allows to complete within broken |
|
1315 |
input that escapes its normal semantic context, e.g.\ antiquotations or |
|
1316 |
string literals in ML, which do not allow arbitrary backslash sequences. |
|
58618 | 1317 |
\<close> |
57325 | 1318 |
|
1319 |
||
58618 | 1320 |
subsection \<open>Input events \label{sec:completion-input}\<close> |
57324 | 1321 |
|
58618 | 1322 |
text \<open> |
57332 | 1323 |
Completion is triggered by certain events produced by the user, with |
1324 |
optional delay after keyboard input according to @{system_option |
|
1325 |
jedit_completion_delay}. |
|
57325 | 1326 |
|
61439 | 1327 |
\<^descr>[Explicit completion] works via action @{action_ref |
57335 | 1328 |
"isabelle.complete"} with keyboard shortcut @{verbatim "C+b"}. This |
1329 |
overrides the shortcut for @{action_ref "complete-word"} in jEdit, but it is |
|
1330 |
possible to restore the original jEdit keyboard mapping of @{action |
|
61477 | 1331 |
"complete-word"} via \<^emph>\<open>Global Options~/ Shortcuts\<close> and invent a |
57335 | 1332 |
different one for @{action "isabelle.complete"}. |
57325 | 1333 |
|
61439 | 1334 |
\<^descr>[Explicit spell-checker completion] works via @{action_ref |
57332 | 1335 |
"isabelle.complete-word"}, which is exposed in the jEdit context menu, if |
1336 |
the mouse points to a word that the spell-checker can complete. |
|
1337 |
||
61439 | 1338 |
\<^descr>[Implicit completion] works via regular keyboard input of the editor. |
57335 | 1339 |
It depends on further side-conditions: |
57325 | 1340 |
|
61458 | 1341 |
\<^enum> The system option @{system_option_ref jedit_completion} needs to |
1342 |
be enabled (default). |
|
57325 | 1343 |
|
61458 | 1344 |
\<^enum> Completion of syntax keywords requires at least 3 relevant |
1345 |
characters in the text. |
|
57325 | 1346 |
|
61458 | 1347 |
\<^enum> The system option @{system_option_ref jedit_completion_delay} |
1348 |
determines an additional delay (0.5 by default), before opening a completion |
|
1349 |
popup. The delay gives the prover a chance to provide semantic completion |
|
1350 |
information, notably the context (\secref{sec:completion-context}). |
|
57325 | 1351 |
|
61458 | 1352 |
\<^enum> The system option @{system_option_ref jedit_completion_immediate} |
1353 |
(enabled by default) controls whether replacement text should be inserted |
|
1354 |
immediately without popup, regardless of @{system_option |
|
1355 |
jedit_completion_delay}. This aggressive mode of completion is restricted to |
|
1356 |
Isabelle symbols and their abbreviations (\secref{sec:symbols}). |
|
57325 | 1357 |
|
61458 | 1358 |
\<^enum> Completion of symbol abbreviations with only one relevant |
1359 |
character in the text always enforces an explicit popup, |
|
1360 |
regardless of @{system_option_ref jedit_completion_immediate}. |
|
58618 | 1361 |
\<close> |
57324 | 1362 |
|
1363 |
||
58618 | 1364 |
subsection \<open>Completion popup \label{sec:completion-popup}\<close> |
57324 | 1365 |
|
58618 | 1366 |
text \<open> |
61477 | 1367 |
A \<^emph>\<open>completion popup\<close> is a minimally invasive GUI component over the |
57335 | 1368 |
text area that offers a selection of completion items to be inserted into |
57420 | 1369 |
the text, e.g.\ by mouse clicks. Items are sorted dynamically, according to |
57833
2c2bae3da1c2
completion popup supports both ENTER and TAB (default);
wenzelm
parents:
57822
diff
changeset
|
1370 |
the frequency of selection, with persistent history. The popup may interpret |
2c2bae3da1c2
completion popup supports both ENTER and TAB (default);
wenzelm
parents:
57822
diff
changeset
|
1371 |
special keys @{verbatim ENTER}, @{verbatim TAB}, @{verbatim ESCAPE}, |
2c2bae3da1c2
completion popup supports both ENTER and TAB (default);
wenzelm
parents:
57822
diff
changeset
|
1372 |
@{verbatim UP}, @{verbatim DOWN}, @{verbatim PAGE_UP}, @{verbatim |
2c2bae3da1c2
completion popup supports both ENTER and TAB (default);
wenzelm
parents:
57822
diff
changeset
|
1373 |
PAGE_DOWN}, but all other key events are passed to the underlying text area. |
2c2bae3da1c2
completion popup supports both ENTER and TAB (default);
wenzelm
parents:
57822
diff
changeset
|
1374 |
This allows to ignore unwanted completions most of the time and continue |
2c2bae3da1c2
completion popup supports both ENTER and TAB (default);
wenzelm
parents:
57822
diff
changeset
|
1375 |
typing quickly. Thus the popup serves as a mechanism of confirmation of |
2c2bae3da1c2
completion popup supports both ENTER and TAB (default);
wenzelm
parents:
57822
diff
changeset
|
1376 |
proposed items, but the default is to continue without completion. |
57324 | 1377 |
|
1378 |
The meaning of special keys is as follows: |
|
1379 |
||
61415 | 1380 |
\<^medskip> |
57324 | 1381 |
\begin{tabular}{ll} |
61477 | 1382 |
\<^bold>\<open>key\<close> & \<^bold>\<open>action\<close> \\\hline |
57833
2c2bae3da1c2
completion popup supports both ENTER and TAB (default);
wenzelm
parents:
57822
diff
changeset
|
1383 |
@{verbatim "ENTER"} & select completion (if @{system_option jedit_completion_select_enter}) \\ |
2c2bae3da1c2
completion popup supports both ENTER and TAB (default);
wenzelm
parents:
57822
diff
changeset
|
1384 |
@{verbatim "TAB"} & select completion (if @{system_option jedit_completion_select_tab}) \\ |
57324 | 1385 |
@{verbatim "ESCAPE"} & dismiss popup \\ |
1386 |
@{verbatim "UP"} & move up one item \\ |
|
1387 |
@{verbatim "DOWN"} & move down one item \\ |
|
1388 |
@{verbatim "PAGE_UP"} & move up one page of items \\ |
|
1389 |
@{verbatim "PAGE_DOWN"} & move down one page of items \\ |
|
1390 |
\end{tabular} |
|
61415 | 1391 |
\<^medskip> |
57324 | 1392 |
|
1393 |
Movement within the popup is only active for multiple items. |
|
1394 |
Otherwise the corresponding key event retains its standard meaning |
|
1395 |
within the underlying text area. |
|
58618 | 1396 |
\<close> |
57324 | 1397 |
|
1398 |
||
58618 | 1399 |
subsection \<open>Insertion \label{sec:completion-insert}\<close> |
57324 | 1400 |
|
58618 | 1401 |
text \<open> |
57333 | 1402 |
Completion may first propose replacements to be selected (via a popup), or |
1403 |
replace text immediately in certain situations and depending on certain |
|
1404 |
options like @{system_option jedit_completion_immediate}. In any case, |
|
57420 | 1405 |
insertion works uniformly, by imitating normal jEdit text insertion, |
61477 | 1406 |
depending on the state of the \<^emph>\<open>text selection\<close>. Isabelle/jEdit tries to |
57420 | 1407 |
accommodate the most common forms of advanced selections in jEdit, but not |
1408 |
all combinations make sense. At least the following important cases are |
|
1409 |
well-defined: |
|
57333 | 1410 |
|
61439 | 1411 |
\<^descr>[No selection.] The original is removed and the replacement inserted, |
57333 | 1412 |
depending on the caret position. |
57324 | 1413 |
|
61439 | 1414 |
\<^descr>[Rectangular selection of zero width.] This special case is treated by |
57333 | 1415 |
jEdit as ``tall caret'' and insertion of completion imitates its normal |
57335 | 1416 |
behaviour: separate copies of the replacement are inserted for each line of |
1417 |
the selection. |
|
57333 | 1418 |
|
61439 | 1419 |
\<^descr>[Other rectangular selection or multiple selections.] Here the original |
57335 | 1420 |
is removed and the replacement is inserted for each line (or segment) of the |
1421 |
selection. |
|
57333 | 1422 |
|
1423 |
||
57335 | 1424 |
Support for multiple selections is particularly useful for |
61477 | 1425 |
\<^emph>\<open>HyperSearch\<close>: clicking on one of the items in the \<^emph>\<open>HyperSearch |
1426 |
Results\<close> window makes jEdit select all its occurrences in the corresponding |
|
57335 | 1427 |
line of text. Then explicit completion can be invoked via @{verbatim "C+b"}, |
61493 | 1428 |
e.g.\ to replace occurrences of @{verbatim "-->"} by \<open>\<longrightarrow>\<close>. |
57333 | 1429 |
|
61415 | 1430 |
\<^medskip> |
1431 |
Insertion works by removing and inserting pieces of text from the |
|
57335 | 1432 |
buffer. This counts as one atomic operation on the jEdit history. Thus |
1433 |
unintended completions may be reverted by the regular @{action undo} action |
|
1434 |
of jEdit. According to normal jEdit policies, the recovered text after |
|
1435 |
@{action undo} is selected: @{verbatim ESCAPE} is required to reset the |
|
1436 |
selection and to continue typing more text. |
|
58618 | 1437 |
\<close> |
57324 | 1438 |
|
1439 |
||
58618 | 1440 |
subsection \<open>Options \label{sec:completion-options}\<close> |
57324 | 1441 |
|
58618 | 1442 |
text \<open> |
57324 | 1443 |
This is a summary of Isabelle/Scala system options that are relevant for |
61477 | 1444 |
completion. They may be configured in \<^emph>\<open>Plugin Options~/ Isabelle~/ |
1445 |
General\<close> as usual. |
|
57332 | 1446 |
|
61415 | 1447 |
\<^item> @{system_option_def completion_limit} specifies the maximum number of |
60257 | 1448 |
items for various semantic completion operations (name-space entries etc.) |
57332 | 1449 |
|
61415 | 1450 |
\<^item> @{system_option_def jedit_completion} guards implicit completion via |
57335 | 1451 |
regular jEdit key events (\secref{sec:completion-input}): it allows to |
1452 |
disable implicit completion altogether. |
|
57324 | 1453 |
|
61415 | 1454 |
\<^item> @{system_option_def jedit_completion_select_enter} and |
57833
2c2bae3da1c2
completion popup supports both ENTER and TAB (default);
wenzelm
parents:
57822
diff
changeset
|
1455 |
@{system_option_def jedit_completion_select_tab} enable keys to select a |
2c2bae3da1c2
completion popup supports both ENTER and TAB (default);
wenzelm
parents:
57822
diff
changeset
|
1456 |
completion item from the popup (\secref{sec:completion-popup}). Note that a |
2c2bae3da1c2
completion popup supports both ENTER and TAB (default);
wenzelm
parents:
57822
diff
changeset
|
1457 |
regular mouse click on the list of items is always possible. |
2c2bae3da1c2
completion popup supports both ENTER and TAB (default);
wenzelm
parents:
57822
diff
changeset
|
1458 |
|
61415 | 1459 |
\<^item> @{system_option_def jedit_completion_context} specifies whether the |
57335 | 1460 |
language context provided by the prover should be used at all. Disabling |
1461 |
that option makes completion less ``semantic''. Note that incomplete or |
|
1462 |
severely broken input may cause some disagreement of the prover and the user |
|
1463 |
about the intended language context. |
|
57332 | 1464 |
|
61415 | 1465 |
\<^item> @{system_option_def jedit_completion_delay} and @{system_option_def |
57333 | 1466 |
jedit_completion_immediate} determine the handling of keyboard events for |
1467 |
implicit completion (\secref{sec:completion-input}). |
|
57332 | 1468 |
|
57333 | 1469 |
A @{system_option jedit_completion_delay}~@{verbatim "> 0"} postpones the |
57335 | 1470 |
processing of key events, until after the user has stopped typing for the |
57333 | 1471 |
given time span, but @{system_option jedit_completion_immediate}~@{verbatim |
1472 |
"= true"} means that abbreviations of Isabelle symbols are handled |
|
1473 |
nonetheless. |
|
57332 | 1474 |
|
61415 | 1475 |
\<^item> @{system_option_def jedit_completion_path_ignore} specifies ``glob'' |
57335 | 1476 |
patterns to ignore in file-system path completion (separated by colons), |
1477 |
e.g.\ backup files ending with tilde. |
|
57332 | 1478 |
|
61415 | 1479 |
\<^item> @{system_option_def spell_checker} is a global guard for all |
57333 | 1480 |
spell-checker operations: it allows to disable that mechanism altogether. |
57332 | 1481 |
|
61415 | 1482 |
\<^item> @{system_option_def spell_checker_dictionary} determines the current |
57335 | 1483 |
dictionary, taken from the colon-separated list in the settings variable |
57333 | 1484 |
@{setting_def JORTHO_DICTIONARIES}. There are jEdit actions to specify local |
1485 |
updates to a dictionary, by including or excluding words. The result of |
|
1486 |
permanent dictionary updates is stored in the directory @{file_unchecked |
|
57335 | 1487 |
"$ISABELLE_HOME_USER/dictionaries"}, in a separate file for each dictionary. |
57332 | 1488 |
|
61415 | 1489 |
\<^item> @{system_option_def spell_checker_elements} specifies a |
57333 | 1490 |
comma-separated list of markup elements that delimit words in the source |
1491 |
that is subject to spell-checking, including various forms of comments. |
|
58618 | 1492 |
\<close> |
54361 | 1493 |
|
1494 |
||
58618 | 1495 |
section \<open>Automatically tried tools \label{sec:auto-tools}\<close> |
54353 | 1496 |
|
58618 | 1497 |
text \<open> |
57325 | 1498 |
Continuous document processing works asynchronously in the background. |
1499 |
Visible document source that has been evaluated may get augmented by |
|
61477 | 1500 |
additional results of \<^emph>\<open>asynchronous print functions\<close>. The canonical |
57325 | 1501 |
example is proof state output, which is always enabled. More heavy-weight |
1502 |
print functions may be applied, in order to prove or disprove parts of the |
|
1503 |
formal text by other means. |
|
54354 | 1504 |
|
1505 |
Isabelle/HOL provides various automatically tried tools that operate |
|
1506 |
on outermost goal statements (e.g.\ @{command lemma}, @{command |
|
1507 |
theorem}), independently of the state of the current proof attempt. |
|
1508 |
They work implicitly without any arguments. Results are output as |
|
61477 | 1509 |
\<^emph>\<open>information messages\<close>, which are indicated in the text area by |
54356 | 1510 |
blue squiggles and a blue information sign in the gutter (see |
1511 |
\figref{fig:auto-tools}). The message content may be shown as for |
|
57316 | 1512 |
other output (see also \secref{sec:output}). Some tools |
61477 | 1513 |
produce output with \<^emph>\<open>sendback\<close> markup, which means that |
54356 | 1514 |
clicking on certain parts of the output inserts that text into the |
1515 |
source in the proper place. |
|
1516 |
||
54357 | 1517 |
\begin{figure}[htb] |
54356 | 1518 |
\begin{center} |
57312 | 1519 |
\includegraphics[scale=0.333]{auto-tools} |
54356 | 1520 |
\end{center} |
57312 | 1521 |
\caption{Result of automatically tried tools} |
54356 | 1522 |
\label{fig:auto-tools} |
1523 |
\end{figure} |
|
54354 | 1524 |
|
61415 | 1525 |
\<^medskip> |
1526 |
The following Isabelle system options control the behavior |
|
54354 | 1527 |
of automatically tried tools (see also the jEdit dialog window |
61477 | 1528 |
\<^emph>\<open>Plugin Options~/ Isabelle~/ General~/ Automatically tried |
1529 |
tools\<close>): |
|
54354 | 1530 |
|
61415 | 1531 |
\<^item> @{system_option_ref auto_methods} controls automatic use of a |
54354 | 1532 |
combination of standard proof methods (@{method auto}, @{method |
54372 | 1533 |
simp}, @{method blast}, etc.). This corresponds to the Isar command |
58554 | 1534 |
@{command_ref "try0"} @{cite "isabelle-isar-ref"}. |
54354 | 1535 |
|
1536 |
The tool is disabled by default, since unparameterized invocation of |
|
1537 |
standard proof methods often consumes substantial CPU resources |
|
1538 |
without leading to success. |
|
1539 |
||
61415 | 1540 |
\<^item> @{system_option_ref auto_nitpick} controls a slightly reduced |
57329 | 1541 |
version of @{command_ref nitpick}, which tests for counterexamples using |
54354 | 1542 |
first-order relational logic. See also the Nitpick manual |
58554 | 1543 |
@{cite "isabelle-nitpick"}. |
54354 | 1544 |
|
1545 |
This tool is disabled by default, due to the extra overhead of |
|
1546 |
invoking an external Java process for each attempt to disprove a |
|
1547 |
subgoal. |
|
1548 |
||
61415 | 1549 |
\<^item> @{system_option_ref auto_quickcheck} controls automatic use of |
57329 | 1550 |
@{command_ref quickcheck}, which tests for counterexamples using a |
54354 | 1551 |
series of assignments for free variables of a subgoal. |
1552 |
||
61477 | 1553 |
This tool is \<^emph>\<open>enabled\<close> by default. It requires little |
54354 | 1554 |
overhead, but is a bit weaker than @{command nitpick}. |
1555 |
||
61415 | 1556 |
\<^item> @{system_option_ref auto_sledgehammer} controls a significantly |
57329 | 1557 |
reduced version of @{command_ref sledgehammer}, which attempts to prove |
54354 | 1558 |
a subgoal using external automatic provers. See also the |
58554 | 1559 |
Sledgehammer manual @{cite "isabelle-sledgehammer"}. |
54354 | 1560 |
|
1561 |
This tool is disabled by default, due to the relatively heavy nature |
|
1562 |
of Sledgehammer. |
|
1563 |
||
61415 | 1564 |
\<^item> @{system_option_ref auto_solve_direct} controls automatic use of |
57329 | 1565 |
@{command_ref solve_direct}, which checks whether the current subgoals |
54354 | 1566 |
can be solved directly by an existing theorem. This also helps to |
1567 |
detect duplicate lemmas. |
|
1568 |
||
61477 | 1569 |
This tool is \<^emph>\<open>enabled\<close> by default. |
54354 | 1570 |
|
1571 |
||
1572 |
Invocation of automatically tried tools is subject to some global |
|
1573 |
policies of parallel execution, which may be configured as follows: |
|
1574 |
||
61415 | 1575 |
\<^item> @{system_option_ref auto_time_limit} (default 2.0) determines the |
54372 | 1576 |
timeout (in seconds) for each tool execution. |
54354 | 1577 |
|
61415 | 1578 |
\<^item> @{system_option_ref auto_time_start} (default 1.0) determines the |
54354 | 1579 |
start delay (in seconds) for automatically tried tools, after the |
1580 |
main command evaluation is finished. |
|
1581 |
||
1582 |
||
1583 |
Each tool is submitted independently to the pool of parallel |
|
1584 |
execution tasks in Isabelle/ML, using hardwired priorities according |
|
1585 |
to its relative ``heaviness''. The main stages of evaluation and |
|
1586 |
printing of proof states take precedence, but an already running |
|
1587 |
tool is not canceled and may thus reduce reactivity of proof |
|
1588 |
document processing. |
|
1589 |
||
1590 |
Users should experiment how the available CPU resources (number of |
|
1591 |
cores) are best invested to get additional feedback from prover in |
|
54372 | 1592 |
the background, by using a selection of weaker or stronger tools. |
58618 | 1593 |
\<close> |
54353 | 1594 |
|
1595 |
||
58618 | 1596 |
section \<open>Sledgehammer \label{sec:sledgehammer}\<close> |
54353 | 1597 |
|
61477 | 1598 |
text \<open>The \<^emph>\<open>Sledgehammer\<close> panel (\figref{fig:sledgehammer}) |
54372 | 1599 |
provides a view on some independent execution of the Isar command |
57329 | 1600 |
@{command_ref sledgehammer}, with process indicator (spinning wheel) and |
54372 | 1601 |
GUI elements for important Sledgehammer arguments and options. Any |
54356 | 1602 |
number of Sledgehammer panels may be active, according to the |
54372 | 1603 |
standard policies of Dockable Window Management in jEdit. Closing |
1604 |
such windows also cancels the corresponding prover tasks. |
|
54356 | 1605 |
|
54357 | 1606 |
\begin{figure}[htb] |
54356 | 1607 |
\begin{center} |
57312 | 1608 |
\includegraphics[scale=0.333]{sledgehammer} |
54356 | 1609 |
\end{center} |
1610 |
\caption{An instance of the Sledgehammer panel} |
|
1611 |
\label{fig:sledgehammer} |
|
1612 |
\end{figure} |
|
54355 | 1613 |
|
61477 | 1614 |
The \<^emph>\<open>Apply\<close> button attaches a fresh invocation of @{command |
54355 | 1615 |
sledgehammer} to the command where the cursor is pointing in the |
1616 |
text --- this should be some pending proof problem. Further buttons |
|
61477 | 1617 |
like \<^emph>\<open>Cancel\<close> and \<^emph>\<open>Locate\<close> help to manage the running |
54355 | 1618 |
process. |
1619 |
||
1620 |
Results appear incrementally in the output window of the panel. |
|
61477 | 1621 |
Proposed proof snippets are marked-up as \<^emph>\<open>sendback\<close>, which |
54355 | 1622 |
means a single mouse click inserts the text into a suitable place of |
1623 |
the original source. Some manual editing may be required |
|
58618 | 1624 |
nonetheless, say to remove earlier proof attempts.\<close> |
54353 | 1625 |
|
1626 |
||
60255
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1627 |
chapter \<open>Isabelle document preparation\<close> |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1628 |
|
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1629 |
text \<open>The ultimate purpose of Isabelle is to produce nicely rendered documents |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1630 |
with the Isabelle document preparation system, which is based on {\LaTeX}; |
60270 | 1631 |
see also @{cite "isabelle-system" and "isabelle-isar-ref"}. Isabelle/jEdit |
60255
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1632 |
provides some additional support for document editing.\<close> |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1633 |
|
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1634 |
|
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1635 |
section \<open>Document outline\<close> |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1636 |
|
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1637 |
text \<open>Theory sources may contain document markup commands, such as |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1638 |
@{command_ref chapter}, @{command_ref section}, @{command subsection}. The |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1639 |
Isabelle SideKick parser (\secref{sec:sidekick}) represents this document |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1640 |
outline as structured tree view, with formal statements and proofs nested |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1641 |
inside; see \figref{fig:sidekick-document}. |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1642 |
|
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1643 |
\begin{figure}[htb] |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1644 |
\begin{center} |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1645 |
\includegraphics[scale=0.333]{sidekick-document} |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1646 |
\end{center} |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1647 |
\caption{Isabelle document outline via SideKick tree view} |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1648 |
\label{fig:sidekick-document} |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1649 |
\end{figure} |
60264 | 1650 |
|
1651 |
It is also possible to use text folding according to this structure, by |
|
61477 | 1652 |
adjusting \<^emph>\<open>Utilities / Buffer Options / Folding mode\<close> of jEdit. The |
60264 | 1653 |
default mode @{verbatim isabelle} uses the structure of formal definitions, |
1654 |
statements, and proofs. The alternative mode @{verbatim sidekick} uses the |
|
1655 |
document structure of the SideKick parser, as explained above.\<close> |
|
1656 |
||
60255
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1657 |
|
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1658 |
section \<open>Citations and Bib{\TeX} entries\<close> |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1659 |
|
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1660 |
text \<open>Citations are managed by {\LaTeX} and Bib{\TeX} in @{verbatim ".bib"} |
60257 | 1661 |
files. The Isabelle session build process and the @{tool latex} tool @{cite |
60270 | 1662 |
"isabelle-system"} are smart enough to assemble the result, based on the |
60257 | 1663 |
session directory layout. |
60255
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1664 |
|
61493 | 1665 |
The document antiquotation \<open>@{cite}\<close> is described in @{cite |
60255
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1666 |
"isabelle-isar-ref"}. Within the Prover IDE it provides semantic markup for |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1667 |
tooltips, hyperlinks, and completion for Bib{\TeX} database entries. |
61477 | 1668 |
Isabelle/jEdit does \<^emph>\<open>not\<close> know about the actual Bib{\TeX} environment |
60255
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1669 |
used in {\LaTeX} batch-mode, but it can take citations from those @{verbatim |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1670 |
".bib"} files that happen to be open in the editor; see |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1671 |
\figref{fig:cite-completion}. |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1672 |
|
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1673 |
\begin{figure}[htb] |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1674 |
\begin{center} |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1675 |
\includegraphics[scale=0.333]{cite-completion} |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1676 |
\end{center} |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1677 |
\caption{Semantic completion of citations from open Bib{\TeX} files} |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1678 |
\label{fig:cite-completion} |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1679 |
\end{figure} |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1680 |
|
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1681 |
Isabelle/jEdit also provides some support for editing @{verbatim ".bib"} |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1682 |
files themselves. There is syntax highlighting based on entry types |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1683 |
(according to standard Bib{\TeX} styles), a context-menu to compose entries |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1684 |
systematically, and a SideKick tree view of the overall content; see |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1685 |
\figref{fig:bibtex-mode}. |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1686 |
|
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1687 |
\begin{figure}[htb] |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1688 |
\begin{center} |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1689 |
\includegraphics[scale=0.333]{bibtex-mode} |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1690 |
\end{center} |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1691 |
\caption{Bib{\TeX} mode with context menu and SideKick tree view} |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1692 |
\label{fig:bibtex-mode} |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1693 |
\end{figure} |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1694 |
\<close> |
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1695 |
|
0466bd194d74
more on Isabelle document preparation and bibtex files;
wenzelm
parents:
58618
diff
changeset
|
1696 |
|
58618 | 1697 |
chapter \<open>Miscellaneous tools\<close> |
54358 | 1698 |
|
58618 | 1699 |
section \<open>Timing\<close> |
54359 | 1700 |
|
58618 | 1701 |
text \<open>Managed evaluation of commands within PIDE documents includes |
54359 | 1702 |
timing information, which consists of elapsed (wall-clock) time, CPU |
1703 |
time, and GC (garbage collection) time. Note that in a |
|
1704 |
multithreaded system it is difficult to measure execution time |
|
1705 |
precisely: elapsed time is closer to the real requirements of |
|
1706 |
runtime resources than CPU or GC time, which are both subject to |
|
1707 |
influences from the parallel environment that are outside the scope |
|
1708 |
of the current command transaction. |
|
1709 |
||
61477 | 1710 |
The \<^emph>\<open>Timing\<close> panel provides an overview of cumulative command |
54359 | 1711 |
timings for each document node. Commands with elapsed time below |
1712 |
the given threshold are ignored in the grand total. Nodes are |
|
1713 |
sorted according to their overall timing. For the document node |
|
1714 |
that corresponds to the current buffer, individual command timings |
|
1715 |
are shown as well. A double-click on a theory node or command moves |
|
1716 |
the editor focus to that particular source position. |
|
1717 |
||
1718 |
It is also possible to reveal individual timing information via some |
|
1719 |
tooltip for the corresponding command keyword, using the technique |
|
1720 |
of mouse hovering with @{verbatim CONTROL}/@{verbatim COMMAND} |
|
1721 |
modifier key as explained in \secref{sec:tooltips-hyperlinks}. |
|
1722 |
Actual display of timing depends on the global option |
|
57329 | 1723 |
@{system_option_ref jedit_timing_threshold}, which can be configured in |
61477 | 1724 |
\<^emph>\<open>Plugin Options~/ Isabelle~/ General\<close>. |
54360 | 1725 |
|
61415 | 1726 |
\<^medskip> |
61477 | 1727 |
The \<^emph>\<open>Monitor\<close> panel visualizes various data collections about |
57869 | 1728 |
recent activity of the Isabelle/ML task farm and the underlying ML runtime |
1729 |
system. The display is continuously updated according to @{system_option_ref |
|
1730 |
editor_chart_delay}. Note that the painting of the chart takes considerable |
|
1731 |
runtime itself --- on the Java Virtual Machine that runs Isabelle/Scala, not |
|
1732 |
Isabelle/ML. Internally, the Isabelle/Scala module @{verbatim |
|
1733 |
isabelle.ML_Statistics} provides further access to statistics of |
|
58618 | 1734 |
Isabelle/ML.\<close> |
54359 | 1735 |
|
1736 |
||
58618 | 1737 |
section \<open>Low-level output\<close> |
54358 | 1738 |
|
58618 | 1739 |
text \<open>Prover output is normally shown directly in the main text area |
61477 | 1740 |
or secondary \<^emph>\<open>Output\<close> panels, as explained in |
57316 | 1741 |
\secref{sec:output}. |
54358 | 1742 |
|
1743 |
Beyond this, it is occasionally useful to inspect low-level output |
|
1744 |
channels via some of the following additional panels: |
|
1745 |
||
61477 | 1746 |
\<^item> \<^emph>\<open>Protocol\<close> shows internal messages between the |
60257 | 1747 |
Isabelle/Scala and Isabelle/ML side of the PIDE document editing protocol. |
54358 | 1748 |
Recording of messages starts with the first activation of the |
1749 |
corresponding dockable window; earlier messages are lost. |
|
1750 |
||
1751 |
Actual display of protocol messages causes considerable slowdown, so |
|
61477 | 1752 |
it is important to undock all \<^emph>\<open>Protocol\<close> panels for production |
54372 | 1753 |
work. |
54358 | 1754 |
|
61477 | 1755 |
\<^item> \<^emph>\<open>Raw Output\<close> shows chunks of text from the @{verbatim |
54358 | 1756 |
stdout} and @{verbatim stderr} channels of the prover process. |
1757 |
Recording of output starts with the first activation of the |
|
1758 |
corresponding dockable window; earlier output is lost. |
|
1759 |
||
1760 |
The implicit stateful nature of physical I/O channels makes it |
|
1761 |
difficult to relate raw output to the actual command from where it |
|
1762 |
was originating. Parallel execution may add to the confusion. |
|
1763 |
Peeking at physical process I/O is only the last resort to diagnose |
|
57310 | 1764 |
problems with tools that are not PIDE compliant. |
54358 | 1765 |
|
57310 | 1766 |
Under normal circumstances, prover output always works via managed message |
1767 |
channels (corresponding to @{ML writeln}, @{ML warning}, @{ML |
|
57420 | 1768 |
Output.error_message} in Isabelle/ML), which are displayed by regular means |
60257 | 1769 |
within the document model (\secref{sec:output}). Unhandled Isabelle/ML |
1770 |
exceptions are printed by the system via @{ML Output.error_message}. |
|
54358 | 1771 |
|
61477 | 1772 |
\<^item> \<^emph>\<open>Syslog\<close> shows system messages that might be relevant to diagnose |
60257 | 1773 |
problems with the startup or shutdown phase of the prover process; this also |
1774 |
includes raw output on @{verbatim stderr}. Isabelle/ML also provides an |
|
1775 |
explicit @{ML Output.system_message} operation, which is occasionally useful |
|
1776 |
for diagnostic purposes within the system infrastructure itself. |
|
54358 | 1777 |
|
1778 |
A limited amount of syslog messages are buffered, independently of |
|
61477 | 1779 |
the docking state of the \<^emph>\<open>Syslog\<close> panel. This allows to |
54358 | 1780 |
diagnose serious problems with Isabelle/PIDE process management, |
1781 |
outside of the actual protocol layer. |
|
1782 |
||
1783 |
Under normal situations, such low-level system output can be |
|
1784 |
ignored. |
|
58618 | 1785 |
\<close> |
54358 | 1786 |
|
1787 |
||
58618 | 1788 |
chapter \<open>Known problems and workarounds \label{sec:problems}\<close> |
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
1789 |
|
58618 | 1790 |
text \<open> |
61477 | 1791 |
\<^item> \<^bold>\<open>Problem:\<close> Odd behavior of some diagnostic commands with |
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
1792 |
global side-effects, like writing a physical file. |
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
1793 |
|
61477 | 1794 |
\<^bold>\<open>Workaround:\<close> Copy/paste complete command text from |
57310 | 1795 |
elsewhere, or disable continuous checking temporarily. |
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
1796 |
|
61477 | 1797 |
\<^item> \<^bold>\<open>Problem:\<close> No direct support to remove document nodes from the |
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
1798 |
collection of theories. |
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
1799 |
|
61477 | 1800 |
\<^bold>\<open>Workaround:\<close> Clear the buffer content of unused files and close |
1801 |
\<^emph>\<open>without\<close> saving changes. |
|
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
1802 |
|
61477 | 1803 |
\<^item> \<^bold>\<open>Problem:\<close> Keyboard shortcuts @{verbatim "C+PLUS"} and |
54330 | 1804 |
@{verbatim "C+MINUS"} for adjusting the editor font size depend on |
1805 |
platform details and national keyboards. |
|
1806 |
||
61477 | 1807 |
\<^bold>\<open>Workaround:\<close> Rebind keys via \<^emph>\<open>Global Options~/ |
1808 |
Shortcuts\<close>. |
|
54330 | 1809 |
|
61477 | 1810 |
\<^item> \<^bold>\<open>Problem:\<close> The Mac OS X key sequence @{verbatim |
1811 |
"COMMAND+COMMA"} for application \<^emph>\<open>Preferences\<close> is in conflict with the |
|
1812 |
jEdit default keyboard shortcut for \<^emph>\<open>Incremental Search Bar\<close> (action |
|
57335 | 1813 |
@{action_ref "quick-search"}). |
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
1814 |
|
61477 | 1815 |
\<^bold>\<open>Workaround:\<close> Rebind key via \<^emph>\<open>Global Options~/ |
1816 |
Shortcuts\<close> according to national keyboard, e.g.\ @{verbatim |
|
54372 | 1817 |
"COMMAND+SLASH"} on English ones. |
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
1818 |
|
61477 | 1819 |
\<^item> \<^bold>\<open>Problem:\<close> Mac OS X system fonts sometimes lead to |
54349 | 1820 |
character drop-outs in the main text area. |
1821 |
||
61477 | 1822 |
\<^bold>\<open>Workaround:\<close> Use the default @{verbatim IsabelleText} font. |
54349 | 1823 |
(Do not install that font on the system.) |
1824 |
||
61477 | 1825 |
\<^item> \<^bold>\<open>Problem:\<close> Some Linux/X11 input methods such as IBus |
54330 | 1826 |
tend to disrupt key event handling of Java/AWT/Swing. |
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
1827 |
|
61477 | 1828 |
\<^bold>\<open>Workaround:\<close> Do not use X11 input methods. Note that environment |
57420 | 1829 |
variable @{verbatim XMODIFIERS} is reset by default within Isabelle |
1830 |
settings. |
|
54329 | 1831 |
|
61477 | 1832 |
\<^item> \<^bold>\<open>Problem:\<close> Some Linux/X11 window managers that are |
54329 | 1833 |
not ``re-parenting'' cause problems with additional windows opened |
54331 | 1834 |
by Java. This affects either historic or neo-minimalistic window |
1835 |
managers like @{verbatim awesome} or @{verbatim xmonad}. |
|
54329 | 1836 |
|
61477 | 1837 |
\<^bold>\<open>Workaround:\<close> Use a regular re-parenting X11 window manager. |
54329 | 1838 |
|
61477 | 1839 |
\<^item> \<^bold>\<open>Problem:\<close> Various forks of Linux/X11 window managers and |
60257 | 1840 |
desktop environments (like Gnome) disrupt the handling of menu popups and |
1841 |
mouse positions of Java/AWT/Swing. |
|
54329 | 1842 |
|
61477 | 1843 |
\<^bold>\<open>Workaround:\<close> Use mainstream versions of Linux desktops. |
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
1844 |
|
61477 | 1845 |
\<^item> \<^bold>\<open>Problem:\<close> Native Windows look-and-feel with global font |
60293 | 1846 |
scaling leads to bad GUI rendering of various tree views. |
60291 | 1847 |
|
61477 | 1848 |
\<^bold>\<open>Workaround:\<close> Use \<^emph>\<open>Metal\<close> look-and-feel and re-adjust its |
60291 | 1849 |
primary and secondary font as explained in \secref{sec:hdpi}. |
1850 |
||
61477 | 1851 |
\<^item> \<^bold>\<open>Problem:\<close> Full-screen mode via jEdit action @{action_ref |
57335 | 1852 |
"toggle-full-screen"} (default keyboard shortcut @{verbatim F11}) works on |
1853 |
Windows, but not on Mac OS X or various Linux/X11 window managers. |
|
54349 | 1854 |
|
61477 | 1855 |
\<^bold>\<open>Workaround:\<close> Use native full-screen control of the window |
54372 | 1856 |
manager (notably on Mac OS X). |
58618 | 1857 |
\<close> |
53770
db362319d766
added/updated material from src/Tools/jEdit/README.html;
wenzelm
parents:
53769
diff
changeset
|
1858 |
|
53769 | 1859 |
end |