author | wenzelm |
Thu, 19 Jun 2014 11:47:46 +0200 | |
changeset 57340 | f6e63c1e5127 |
parent 56579 | 4c94f631c595 |
child 57342 | 1dc320dc2ada |
permissions | -rw-r--r-- |
29755 | 1 |
theory Isar |
2 |
imports Base |
|
3 |
begin |
|
20472 | 4 |
|
29759 | 5 |
chapter {* Isar language elements *} |
6 |
||
40126 | 7 |
text {* The Isar proof language (see also |
8 |
\cite[\S2]{isabelle-isar-ref}) consists of three main categories of |
|
57340 | 9 |
language elements: |
29759 | 10 |
|
11 |
\begin{enumerate} |
|
12 |
||
39842 | 13 |
\item Proof \emph{commands} define the primary language of |
14 |
transactions of the underlying Isar/VM interpreter. Typical |
|
15 |
examples are @{command "fix"}, @{command "assume"}, @{command |
|
39844 | 16 |
"show"}, @{command "proof"}, and @{command "qed"}. |
39842 | 17 |
|
39844 | 18 |
Composing proof commands according to the rules of the Isar/VM leads |
19 |
to expressions of structured proof text, such that both the machine |
|
20 |
and the human reader can give it a meaning as formal reasoning. |
|
20472 | 21 |
|
39842 | 22 |
\item Proof \emph{methods} define a secondary language of mixed |
23 |
forward-backward refinement steps involving facts and goals. |
|
39846 | 24 |
Typical examples are @{method rule}, @{method unfold}, and @{method |
39844 | 25 |
simp}. |
29759 | 26 |
|
39842 | 27 |
Methods can occur in certain well-defined parts of the Isar proof |
28 |
language, say as arguments to @{command "proof"}, @{command "qed"}, |
|
29 |
or @{command "by"}. |
|
30 |
||
31 |
\item \emph{Attributes} define a tertiary language of small |
|
39849 | 32 |
annotations to theorems being defined or referenced. Attributes can |
33 |
modify both the context and the theorem. |
|
39842 | 34 |
|
39849 | 35 |
Typical examples are @{attribute intro} (which affects the context), |
36 |
and @{attribute symmetric} (which affects the theorem). |
|
29759 | 37 |
|
38 |
\end{enumerate} |
|
39 |
*} |
|
40 |
||
41 |
||
42 |
section {* Proof commands *} |
|
20520 | 43 |
|
39849 | 44 |
text {* A \emph{proof command} is state transition of the Isar/VM |
45 |
proof interpreter. |
|
46 |
||
40126 | 47 |
In principle, Isar proof commands could be defined in user-space as |
48 |
well. The system is built like that in the first place: one part of |
|
49 |
the commands are primitive, the other part is defined as derived |
|
50 |
elements. Adding to the genuine structured proof language requires |
|
51 |
profound understanding of the Isar/VM machinery, though, so this is |
|
52 |
beyond the scope of this manual. |
|
39842 | 53 |
|
54 |
What can be done realistically is to define some diagnostic commands |
|
39844 | 55 |
that inspect the general state of the Isar/VM, and report some |
56 |
feedback to the user. Typically this involves checking of the |
|
39842 | 57 |
linguistic \emph{mode} of a proof state, or peeking at the pending |
58 |
goals (if available). |
|
39845 | 59 |
|
60 |
Another common application is to define a toplevel command that |
|
40126 | 61 |
poses a problem to the user as Isar proof state and processes the |
62 |
final result relatively to the context. Thus a proof can be |
|
39845 | 63 |
incorporated into the context of some user-space tool, without |
40126 | 64 |
modifying the Isar proof language itself. *} |
39842 | 65 |
|
66 |
text %mlref {* |
|
67 |
\begin{mldecls} |
|
68 |
@{index_ML_type Proof.state} \\ |
|
69 |
@{index_ML Proof.assert_forward: "Proof.state -> Proof.state"} \\ |
|
70 |
@{index_ML Proof.assert_chain: "Proof.state -> Proof.state"} \\ |
|
71 |
@{index_ML Proof.assert_backward: "Proof.state -> Proof.state"} \\ |
|
72 |
@{index_ML Proof.simple_goal: "Proof.state -> {context: Proof.context, goal: thm}"} \\ |
|
73 |
@{index_ML Proof.goal: "Proof.state -> |
|
74 |
{context: Proof.context, facts: thm list, goal: thm}"} \\ |
|
75 |
@{index_ML Proof.raw_goal: "Proof.state -> |
|
76 |
{context: Proof.context, facts: thm list, goal: thm}"} \\ |
|
39845 | 77 |
@{index_ML Proof.theorem: "Method.text option -> |
78 |
(thm list list -> Proof.context -> Proof.context) -> |
|
79 |
(term * term list) list list -> Proof.context -> Proof.state"} \\ |
|
39842 | 80 |
\end{mldecls} |
81 |
||
82 |
\begin{description} |
|
83 |
||
39864 | 84 |
\item Type @{ML_type Proof.state} represents Isar proof states. |
85 |
This is a block-structured configuration with proof context, |
|
86 |
linguistic mode, and optional goal. The latter consists of goal |
|
87 |
context, goal facts (``@{text "using"}''), and tactical goal state |
|
88 |
(see \secref{sec:tactical-goals}). |
|
39842 | 89 |
|
90 |
The general idea is that the facts shall contribute to the |
|
39844 | 91 |
refinement of some parts of the tactical goal --- how exactly is |
92 |
defined by the proof method that is applied in that situation. |
|
39842 | 93 |
|
94 |
\item @{ML Proof.assert_forward}, @{ML Proof.assert_chain}, @{ML |
|
95 |
Proof.assert_backward} are partial identity functions that fail |
|
96 |
unless a certain linguistic mode is active, namely ``@{text |
|
97 |
"proof(state)"}'', ``@{text "proof(chain)"}'', ``@{text |
|
98 |
"proof(prove)"}'', respectively (using the terminology of |
|
99 |
\cite{isabelle-isar-ref}). |
|
100 |
||
101 |
It is advisable study the implementations of existing proof commands |
|
102 |
for suitable modes to be asserted. |
|
103 |
||
104 |
\item @{ML Proof.simple_goal}~@{text "state"} returns the structured |
|
105 |
Isar goal (if available) in the form seen by ``simple'' methods |
|
39846 | 106 |
(like @{method simp} or @{method blast}). The Isar goal facts are |
39842 | 107 |
already inserted as premises into the subgoals, which are presented |
39844 | 108 |
individually as in @{ML Proof.goal}. |
39842 | 109 |
|
110 |
\item @{ML Proof.goal}~@{text "state"} returns the structured Isar |
|
111 |
goal (if available) in the form seen by regular methods (like |
|
112 |
@{method rule}). The auxiliary internal encoding of Pure |
|
113 |
conjunctions is split into individual subgoals as usual. |
|
114 |
||
115 |
\item @{ML Proof.raw_goal}~@{text "state"} returns the structured |
|
116 |
Isar goal (if available) in the raw internal form seen by ``raw'' |
|
39846 | 117 |
methods (like @{method induct}). This form is rarely appropriate |
56579 | 118 |
for diagnostic tools; @{ML Proof.simple_goal} or @{ML Proof.goal} |
39846 | 119 |
should be used in most situations. |
39842 | 120 |
|
39845 | 121 |
\item @{ML Proof.theorem}~@{text "before_qed after_qed statement ctxt"} |
122 |
initializes a toplevel Isar proof state within a given context. |
|
123 |
||
124 |
The optional @{text "before_qed"} method is applied at the end of |
|
125 |
the proof, just before extracting the result (this feature is rarely |
|
126 |
used). |
|
127 |
||
128 |
The @{text "after_qed"} continuation receives the extracted result |
|
129 |
in order to apply it to the final context in a suitable way (e.g.\ |
|
130 |
storing named facts). Note that at this generic level the target |
|
131 |
context is specified as @{ML_type Proof.context}, but the usual |
|
132 |
wrapping of toplevel proofs into command transactions will provide a |
|
40126 | 133 |
@{ML_type local_theory} here (\chref{ch:local-theory}). This |
134 |
affects the way how results are stored. |
|
39845 | 135 |
|
136 |
The @{text "statement"} is given as a nested list of terms, each |
|
137 |
associated with optional @{keyword "is"} patterns as usual in the |
|
40126 | 138 |
Isar source language. The original nested list structure over terms |
139 |
is turned into one over theorems when @{text "after_qed"} is |
|
140 |
invoked. |
|
39845 | 141 |
|
39842 | 142 |
\end{description} |
143 |
*} |
|
144 |
||
20520 | 145 |
|
39843 | 146 |
text %mlantiq {* |
147 |
\begin{matharray}{rcl} |
|
148 |
@{ML_antiquotation_def "Isar.goal"} & : & @{text ML_antiquotation} \\ |
|
149 |
\end{matharray} |
|
150 |
||
151 |
\begin{description} |
|
152 |
||
153 |
\item @{text "@{Isar.goal}"} refers to the regular goal state (if |
|
154 |
available) of the current proof state managed by the Isar toplevel |
|
155 |
--- as abstract value. |
|
156 |
||
157 |
This only works for diagnostic ML commands, such as @{command |
|
158 |
ML_val} or @{command ML_command}. |
|
159 |
||
160 |
\end{description} |
|
161 |
*} |
|
162 |
||
163 |
text %mlex {* The following example peeks at a certain goal configuration. *} |
|
164 |
||
40964 | 165 |
notepad |
166 |
begin |
|
39846 | 167 |
have A and B and C |
39866
5ec01d5acd0c
more robust examples: explicit @{assert} instead of unchecked output;
wenzelm
parents:
39865
diff
changeset
|
168 |
ML_val {* |
5ec01d5acd0c
more robust examples: explicit @{assert} instead of unchecked output;
wenzelm
parents:
39865
diff
changeset
|
169 |
val n = Thm.nprems_of (#goal @{Isar.goal}); |
5ec01d5acd0c
more robust examples: explicit @{assert} instead of unchecked output;
wenzelm
parents:
39865
diff
changeset
|
170 |
@{assert} (n = 3); |
5ec01d5acd0c
more robust examples: explicit @{assert} instead of unchecked output;
wenzelm
parents:
39865
diff
changeset
|
171 |
*} |
39843 | 172 |
oops |
173 |
||
39861
b8d89db3e238
use continental paragraph style, which works better with mixture of (in)formal text;
wenzelm
parents:
39851
diff
changeset
|
174 |
text {* Here we see 3 individual subgoals in the same way as regular |
b8d89db3e238
use continental paragraph style, which works better with mixture of (in)formal text;
wenzelm
parents:
39851
diff
changeset
|
175 |
proof methods would do. *} |
39843 | 176 |
|
20520 | 177 |
|
20472 | 178 |
section {* Proof methods *} |
179 |
||
39847 | 180 |
text {* A @{text "method"} is a function @{text "context \<rightarrow> thm\<^sup>* \<rightarrow> goal |
181 |
\<rightarrow> (cases \<times> goal)\<^sup>*\<^sup>*"} that operates on the full Isar goal |
|
182 |
configuration with context, goal facts, and tactical goal state and |
|
39843 | 183 |
enumerates possible follow-up goal states, with the potential |
39844 | 184 |
addition of named extensions of the proof context (\emph{cases}). |
39847 | 185 |
The latter feature is rarely used. |
186 |
||
187 |
This means a proof method is like a structurally enhanced tactic |
|
188 |
(cf.\ \secref{sec:tactics}). The well-formedness conditions for |
|
189 |
tactics need to hold for methods accordingly, with the following |
|
190 |
additions. |
|
191 |
||
192 |
\begin{itemize} |
|
193 |
||
57340 | 194 |
\item Goal addressing is further limited either to operate |
39847 | 195 |
uniformly on \emph{all} subgoals, or specifically on the |
196 |
\emph{first} subgoal. |
|
197 |
||
198 |
Exception: old-style tactic emulations that are embedded into the |
|
199 |
method space, e.g.\ @{method rule_tac}. |
|
200 |
||
201 |
\item A non-trivial method always needs to make progress: an |
|
202 |
identical follow-up goal state has to be avoided.\footnote{This |
|
203 |
enables the user to write method expressions like @{text "meth\<^sup>+"} |
|
204 |
without looping, while the trivial do-nothing case can be recovered |
|
205 |
via @{text "meth\<^sup>?"}.} |
|
206 |
||
207 |
Exception: trivial stuttering steps, such as ``@{method -}'' or |
|
208 |
@{method succeed}. |
|
209 |
||
210 |
\item Goal facts passed to the method must not be ignored. If there |
|
211 |
is no sensible use of facts outside the goal state, facts should be |
|
212 |
inserted into the subgoals that are addressed by the method. |
|
213 |
||
214 |
\end{itemize} |
|
215 |
||
40126 | 216 |
\medskip Syntactically, the language of proof methods appears as |
217 |
arguments to Isar commands like @{command "by"} or @{command apply}. |
|
218 |
User-space additions are reasonably easy by plugging suitable |
|
219 |
method-valued parser functions into the framework, using the |
|
220 |
@{command method_setup} command, for example. |
|
39843 | 221 |
|
39844 | 222 |
To get a better idea about the range of possibilities, consider the |
40126 | 223 |
following Isar proof schemes. This is the general form of |
224 |
structured proof text: |
|
39843 | 225 |
|
226 |
\medskip |
|
227 |
\begin{tabular}{l} |
|
228 |
@{command from}~@{text "facts\<^sub>1"}~@{command have}~@{text "props"}~@{command using}~@{text "facts\<^sub>2"} \\ |
|
229 |
@{command proof}~@{text "(initial_method)"} \\ |
|
230 |
\quad@{text "body"} \\ |
|
231 |
@{command qed}~@{text "(terminal_method)"} \\ |
|
232 |
\end{tabular} |
|
233 |
\medskip |
|
234 |
||
40126 | 235 |
The goal configuration consists of @{text "facts\<^sub>1"} and |
236 |
@{text "facts\<^sub>2"} appended in that order, and various @{text |
|
237 |
"props"} being claimed. The @{text "initial_method"} is invoked |
|
238 |
with facts and goals together and refines the problem to something |
|
239 |
that is handled recursively in the proof @{text "body"}. The @{text |
|
240 |
"terminal_method"} has another chance to finish any remaining |
|
39843 | 241 |
subgoals, but it does not see the facts of the initial step. |
242 |
||
40126 | 243 |
\medskip This pattern illustrates unstructured proof scripts: |
39843 | 244 |
|
39844 | 245 |
\medskip |
39843 | 246 |
\begin{tabular}{l} |
247 |
@{command have}~@{text "props"} \\ |
|
39844 | 248 |
\quad@{command using}~@{text "facts\<^sub>1"}~@{command apply}~@{text "method\<^sub>1"} \\ |
39843 | 249 |
\quad@{command apply}~@{text "method\<^sub>2"} \\ |
39844 | 250 |
\quad@{command using}~@{text "facts\<^sub>3"}~@{command apply}~@{text "method\<^sub>3"} \\ |
39843 | 251 |
\quad@{command done} \\ |
252 |
\end{tabular} |
|
253 |
\medskip |
|
254 |
||
40126 | 255 |
The @{text "method\<^sub>1"} operates on the original claim while |
39861
b8d89db3e238
use continental paragraph style, which works better with mixture of (in)formal text;
wenzelm
parents:
39851
diff
changeset
|
256 |
using @{text "facts\<^sub>1"}. Since the @{command apply} command |
40126 | 257 |
structurally resets the facts, the @{text "method\<^sub>2"} will |
258 |
operate on the remaining goal state without facts. The @{text |
|
259 |
"method\<^sub>3"} will see again a collection of @{text |
|
260 |
"facts\<^sub>3"} that has been inserted into the script explicitly. |
|
39843 | 261 |
|
40126 | 262 |
\medskip Empirically, any Isar proof method can be categorized as |
39847 | 263 |
follows. |
39843 | 264 |
|
265 |
\begin{enumerate} |
|
266 |
||
39847 | 267 |
\item \emph{Special method with cases} with named context additions |
268 |
associated with the follow-up goal state. |
|
39843 | 269 |
|
39847 | 270 |
Example: @{method "induct"}, which is also a ``raw'' method since it |
271 |
operates on the internal representation of simultaneous claims as |
|
46134 | 272 |
Pure conjunction (\secref{sec:logic-aux}), instead of separate |
273 |
subgoals (\secref{sec:tactical-goals}). |
|
39843 | 274 |
|
39847 | 275 |
\item \emph{Structured method} with strong emphasis on facts outside |
276 |
the goal state. |
|
277 |
||
278 |
Example: @{method "rule"}, which captures the key ideas behind |
|
57340 | 279 |
structured reasoning in Isar in its purest form. |
39843 | 280 |
|
39847 | 281 |
\item \emph{Simple method} with weaker emphasis on facts, which are |
57340 | 282 |
inserted into subgoals to emulate old-style tactical ``premises''. |
39843 | 283 |
|
39847 | 284 |
Examples: @{method "simp"}, @{method "blast"}, @{method "auto"}. |
39843 | 285 |
|
39847 | 286 |
\item \emph{Old-style tactic emulation} with detailed numeric goal |
287 |
addressing and explicit references to entities of the internal goal |
|
288 |
state (which are otherwise invisible from proper Isar proof text). |
|
40126 | 289 |
The naming convention @{text "foo_tac"} makes this special |
290 |
non-standard status clear. |
|
39843 | 291 |
|
39847 | 292 |
Example: @{method "rule_tac"}. |
39843 | 293 |
|
294 |
\end{enumerate} |
|
295 |
||
39847 | 296 |
When implementing proof methods, it is advisable to study existing |
297 |
implementations carefully and imitate the typical ``boiler plate'' |
|
298 |
for context-sensitive parsing and further combinators to wrap-up |
|
39848 | 299 |
tactic expressions as methods.\footnote{Aliases or abbreviations of |
300 |
the standard method combinators should be avoided. Note that from |
|
301 |
Isabelle99 until Isabelle2009 the system did provide various odd |
|
57340 | 302 |
combinations of method syntax wrappers that made applications more |
39848 | 303 |
complicated than necessary.} |
39847 | 304 |
*} |
305 |
||
306 |
text %mlref {* |
|
307 |
\begin{mldecls} |
|
308 |
@{index_ML_type Proof.method} \\ |
|
309 |
@{index_ML METHOD_CASES: "(thm list -> cases_tactic) -> Proof.method"} \\ |
|
310 |
@{index_ML METHOD: "(thm list -> tactic) -> Proof.method"} \\ |
|
311 |
@{index_ML SIMPLE_METHOD: "tactic -> Proof.method"} \\ |
|
312 |
@{index_ML SIMPLE_METHOD': "(int -> tactic) -> Proof.method"} \\ |
|
313 |
@{index_ML Method.insert_tac: "thm list -> int -> tactic"} \\ |
|
314 |
@{index_ML Method.setup: "binding -> (Proof.context -> Proof.method) context_parser -> |
|
315 |
string -> theory -> theory"} \\ |
|
316 |
\end{mldecls} |
|
317 |
||
318 |
\begin{description} |
|
319 |
||
39864 | 320 |
\item Type @{ML_type Proof.method} represents proof methods as |
321 |
abstract type. |
|
39847 | 322 |
|
323 |
\item @{ML METHOD_CASES}~@{text "(fn facts => cases_tactic)"} wraps |
|
324 |
@{text cases_tactic} depending on goal facts as proof method with |
|
325 |
cases; the goal context is passed via method syntax. |
|
326 |
||
327 |
\item @{ML METHOD}~@{text "(fn facts => tactic)"} wraps @{text |
|
328 |
tactic} depending on goal facts as regular proof method; the goal |
|
329 |
context is passed via method syntax. |
|
330 |
||
331 |
\item @{ML SIMPLE_METHOD}~@{text "tactic"} wraps a tactic that |
|
332 |
addresses all subgoals uniformly as simple proof method. Goal facts |
|
333 |
are already inserted into all subgoals before @{text "tactic"} is |
|
334 |
applied. |
|
335 |
||
336 |
\item @{ML SIMPLE_METHOD'}~@{text "tactic"} wraps a tactic that |
|
46267 | 337 |
addresses a specific subgoal as simple proof method that operates on |
338 |
subgoal 1. Goal facts are inserted into the subgoal then the @{text |
|
339 |
"tactic"} is applied. |
|
39847 | 340 |
|
341 |
\item @{ML Method.insert_tac}~@{text "facts i"} inserts @{text |
|
342 |
"facts"} into subgoal @{text "i"}. This is convenient to reproduce |
|
343 |
part of the @{ML SIMPLE_METHOD} or @{ML SIMPLE_METHOD'} wrapping |
|
344 |
within regular @{ML METHOD}, for example. |
|
345 |
||
346 |
\item @{ML Method.setup}~@{text "name parser description"} provides |
|
39848 | 347 |
the functionality of the Isar command @{command method_setup} as ML |
348 |
function. |
|
39847 | 349 |
|
350 |
\end{description} |
|
351 |
*} |
|
352 |
||
39851 | 353 |
text %mlex {* See also @{command method_setup} in |
354 |
\cite{isabelle-isar-ref} which includes some abstract examples. |
|
355 |
||
356 |
\medskip The following toy examples illustrate how the goal facts |
|
56579 | 357 |
and state are passed to proof methods. The predefined proof method |
39848 | 358 |
called ``@{method tactic}'' wraps ML source of type @{ML_type |
40149
4c35be108990
proper markup of uninterpreted ML text as @{ML_text}, not @{verbatim};
wenzelm
parents:
40126
diff
changeset
|
359 |
tactic} (abstracted over @{ML_text facts}). This allows immediate |
39848 | 360 |
experimentation without parsing of concrete syntax. *} |
20472 | 361 |
|
40964 | 362 |
notepad |
363 |
begin |
|
57340 | 364 |
fix A B :: bool |
39847 | 365 |
assume a: A and b: B |
366 |
||
367 |
have "A \<and> B" |
|
57340 | 368 |
apply (tactic \<open>rtac @{thm conjI} 1\<close>) |
369 |
using a apply (tactic \<open>resolve_tac facts 1\<close>) |
|
370 |
using b apply (tactic \<open>resolve_tac facts 1\<close>) |
|
39847 | 371 |
done |
372 |
||
373 |
have "A \<and> B" |
|
374 |
using a and b |
|
57340 | 375 |
ML_val \<open>@{Isar.goal}\<close> |
376 |
apply (tactic \<open>Method.insert_tac facts 1\<close>) |
|
377 |
apply (tactic \<open>(rtac @{thm conjI} THEN_ALL_NEW atac) 1\<close>) |
|
39847 | 378 |
done |
40964 | 379 |
end |
39847 | 380 |
|
39848 | 381 |
text {* \medskip The next example implements a method that simplifies |
57340 | 382 |
the first subgoal by rewrite rules that are given as arguments. *} |
39848 | 383 |
|
57340 | 384 |
method_setup my_simp = |
385 |
\<open>Attrib.thms >> (fn thms => fn ctxt => |
|
39848 | 386 |
SIMPLE_METHOD' (fn i => |
387 |
CHANGED (asm_full_simp_tac |
|
57340 | 388 |
(put_simpset HOL_basic_ss ctxt addsimps thms) i)))\<close> |
389 |
"rewrite subgoal by given rules" |
|
39848 | 390 |
|
391 |
text {* The concrete syntax wrapping of @{command method_setup} always |
|
392 |
passes-through the proof context at the end of parsing, but it is |
|
393 |
not used in this example. |
|
394 |
||
395 |
The @{ML Attrib.thms} parser produces a list of theorems from the |
|
396 |
usual Isar syntax involving attribute expressions etc.\ (syntax |
|
40126 | 397 |
category @{syntax thmrefs}) \cite{isabelle-isar-ref}. The resulting |
40149
4c35be108990
proper markup of uninterpreted ML text as @{ML_text}, not @{verbatim};
wenzelm
parents:
40126
diff
changeset
|
398 |
@{ML_text thms} are added to @{ML HOL_basic_ss} which already |
40126 | 399 |
contains the basic Simplifier setup for HOL. |
39848 | 400 |
|
401 |
The tactic @{ML asm_full_simp_tac} is the one that is also used in |
|
402 |
method @{method simp} by default. The extra wrapping by the @{ML |
|
403 |
CHANGED} tactical ensures progress of simplification: identical goal |
|
404 |
states are filtered out explicitly to make the raw tactic conform to |
|
405 |
standard Isar method behaviour. |
|
406 |
||
407 |
\medskip Method @{method my_simp} can be used in Isar proofs like |
|
408 |
this: |
|
39847 | 409 |
*} |
410 |
||
40964 | 411 |
notepad |
412 |
begin |
|
57340 | 413 |
fix a b c :: 'a |
39851 | 414 |
assume a: "a = b" |
415 |
assume b: "b = c" |
|
416 |
have "a = c" by (my_simp a b) |
|
40964 | 417 |
end |
39851 | 418 |
|
419 |
text {* Here is a similar method that operates on all subgoals, |
|
420 |
instead of just the first one. *} |
|
421 |
||
57340 | 422 |
method_setup my_simp_all = |
423 |
\<open>Attrib.thms >> (fn thms => fn ctxt => |
|
39851 | 424 |
SIMPLE_METHOD |
425 |
(CHANGED |
|
426 |
(ALLGOALS (asm_full_simp_tac |
|
57340 | 427 |
(put_simpset HOL_basic_ss ctxt addsimps thms)))))\<close> |
428 |
"rewrite all subgoals by given rules" |
|
39851 | 429 |
|
40964 | 430 |
notepad |
431 |
begin |
|
57340 | 432 |
fix a b c :: 'a |
39851 | 433 |
assume a: "a = b" |
434 |
assume b: "b = c" |
|
435 |
have "a = c" and "c = b" by (my_simp_all a b) |
|
40964 | 436 |
end |
39848 | 437 |
|
438 |
text {* \medskip Apart from explicit arguments, common proof methods |
|
439 |
typically work with a default configuration provided by the context. |
|
57340 | 440 |
As a shortcut to rule management we use a cheap solution via the |
441 |
functor @{ML_functor Named_Thms} (see also @{file |
|
39848 | 442 |
"~~/src/Pure/Tools/named_thms.ML"}). *} |
443 |
||
39847 | 444 |
ML {* |
445 |
structure My_Simps = |
|
57340 | 446 |
Named_Thms( |
447 |
val name = @{binding my_simp} |
|
448 |
val description = "my_simp rule" |
|
449 |
) |
|
39847 | 450 |
*} |
451 |
setup My_Simps.setup |
|
452 |
||
39861
b8d89db3e238
use continental paragraph style, which works better with mixture of (in)formal text;
wenzelm
parents:
39851
diff
changeset
|
453 |
text {* This provides ML access to a list of theorems in canonical |
b8d89db3e238
use continental paragraph style, which works better with mixture of (in)formal text;
wenzelm
parents:
39851
diff
changeset
|
454 |
declaration order via @{ML My_Simps.get}. The user can add or |
b8d89db3e238
use continental paragraph style, which works better with mixture of (in)formal text;
wenzelm
parents:
39851
diff
changeset
|
455 |
delete rules via the attribute @{attribute my_simp}. The actual |
b8d89db3e238
use continental paragraph style, which works better with mixture of (in)formal text;
wenzelm
parents:
39851
diff
changeset
|
456 |
proof method is now defined as before, but we append the explicit |
b8d89db3e238
use continental paragraph style, which works better with mixture of (in)formal text;
wenzelm
parents:
39851
diff
changeset
|
457 |
arguments and the rules from the context. *} |
39847 | 458 |
|
57340 | 459 |
method_setup my_simp' = |
460 |
\<open>Attrib.thms >> (fn thms => fn ctxt => |
|
39847 | 461 |
SIMPLE_METHOD' (fn i => |
462 |
CHANGED (asm_full_simp_tac |
|
51717
9e7d1c139569
simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents:
48985
diff
changeset
|
463 |
(put_simpset HOL_basic_ss ctxt |
57340 | 464 |
addsimps (thms @ My_Simps.get ctxt)) i)))\<close> |
465 |
"rewrite subgoal by given rules and my_simp rules from the context" |
|
39847 | 466 |
|
39848 | 467 |
text {* |
468 |
\medskip Method @{method my_simp'} can be used in Isar proofs |
|
469 |
like this: |
|
470 |
*} |
|
39847 | 471 |
|
40964 | 472 |
notepad |
473 |
begin |
|
39847 | 474 |
fix a b c |
475 |
assume [my_simp]: "a \<equiv> b" |
|
476 |
assume [my_simp]: "b \<equiv> c" |
|
39848 | 477 |
have "a \<equiv> c" by my_simp' |
40964 | 478 |
end |
39847 | 479 |
|
39851 | 480 |
text {* \medskip The @{method my_simp} variants defined above are |
481 |
``simple'' methods, i.e.\ the goal facts are merely inserted as goal |
|
482 |
premises by the @{ML SIMPLE_METHOD'} or @{ML SIMPLE_METHOD} wrapper. |
|
483 |
For proof methods that are similar to the standard collection of |
|
40126 | 484 |
@{method simp}, @{method blast}, @{method fast}, @{method auto} |
485 |
there is little more that can be done. |
|
39847 | 486 |
|
487 |
Note that using the primary goal facts in the same manner as the |
|
39848 | 488 |
method arguments obtained via concrete syntax or the context does |
489 |
not meet the requirement of ``strong emphasis on facts'' of regular |
|
490 |
proof methods, because rewrite rules as used above can be easily |
|
491 |
ignored. A proof text ``@{command using}~@{text "foo"}~@{command |
|
492 |
"by"}~@{text "my_simp"}'' where @{text "foo"} is not used would |
|
493 |
deceive the reader. |
|
39847 | 494 |
|
495 |
\medskip The technical treatment of rules from the context requires |
|
496 |
further attention. Above we rebuild a fresh @{ML_type simpset} from |
|
39848 | 497 |
the arguments and \emph{all} rules retrieved from the context on |
498 |
every invocation of the method. This does not scale to really large |
|
499 |
collections of rules, which easily emerges in the context of a big |
|
500 |
theory library, for example. |
|
39847 | 501 |
|
39848 | 502 |
This is an inherent limitation of the simplistic rule management via |
503 |
functor @{ML_functor Named_Thms}, because it lacks tool-specific |
|
39847 | 504 |
storage and retrieval. More realistic applications require |
505 |
efficient index-structures that organize theorems in a customized |
|
506 |
manner, such as a discrimination net that is indexed by the |
|
39848 | 507 |
left-hand sides of rewrite rules. For variations on the Simplifier, |
508 |
re-use of the existing type @{ML_type simpset} is adequate, but |
|
40126 | 509 |
scalability would require it be maintained statically within the |
510 |
context data, not dynamically on each tool invocation. *} |
|
39847 | 511 |
|
29759 | 512 |
|
39865 | 513 |
section {* Attributes \label{sec:attributes} *} |
20472 | 514 |
|
39849 | 515 |
text {* An \emph{attribute} is a function @{text "context \<times> thm \<rightarrow> |
516 |
context \<times> thm"}, which means both a (generic) context and a theorem |
|
45414 | 517 |
can be modified simultaneously. In practice this mixed form is very |
518 |
rare, instead attributes are presented either as \emph{declaration |
|
519 |
attribute:} @{text "thm \<rightarrow> context \<rightarrow> context"} or \emph{rule |
|
520 |
attribute:} @{text "context \<rightarrow> thm \<rightarrow> thm"}. |
|
39849 | 521 |
|
522 |
Attributes can have additional arguments via concrete syntax. There |
|
523 |
is a collection of context-sensitive parsers for various logical |
|
524 |
entities (types, terms, theorems). These already take care of |
|
525 |
applying morphisms to the arguments when attribute expressions are |
|
526 |
moved into a different context (see also \secref{sec:morphisms}). |
|
527 |
||
528 |
When implementing declaration attributes, it is important to operate |
|
529 |
exactly on the variant of the generic context that is provided by |
|
530 |
the system, which is either global theory context or local proof |
|
531 |
context. In particular, the background theory of a local context |
|
532 |
must not be modified in this situation! *} |
|
533 |
||
534 |
text %mlref {* |
|
535 |
\begin{mldecls} |
|
45414 | 536 |
@{index_ML_type attribute} \\ |
39849 | 537 |
@{index_ML Thm.rule_attribute: "(Context.generic -> thm -> thm) -> attribute"} \\ |
538 |
@{index_ML Thm.declaration_attribute: " |
|
539 |
(thm -> Context.generic -> Context.generic) -> attribute"} \\ |
|
540 |
@{index_ML Attrib.setup: "binding -> attribute context_parser -> |
|
541 |
string -> theory -> theory"} \\ |
|
542 |
\end{mldecls} |
|
543 |
||
544 |
\begin{description} |
|
545 |
||
39864 | 546 |
\item Type @{ML_type attribute} represents attributes as concrete |
547 |
type alias. |
|
39849 | 548 |
|
549 |
\item @{ML Thm.rule_attribute}~@{text "(fn context => rule)"} wraps |
|
550 |
a context-dependent rule (mapping on @{ML_type thm}) as attribute. |
|
551 |
||
552 |
\item @{ML Thm.declaration_attribute}~@{text "(fn thm => decl)"} |
|
553 |
wraps a theorem-dependent declaration (mapping on @{ML_type |
|
554 |
Context.generic}) as attribute. |
|
555 |
||
556 |
\item @{ML Attrib.setup}~@{text "name parser description"} provides |
|
557 |
the functionality of the Isar command @{command attribute_setup} as |
|
558 |
ML function. |
|
559 |
||
560 |
\end{description} |
|
561 |
*} |
|
562 |
||
45592 | 563 |
text %mlantiq {* |
564 |
\begin{matharray}{rcl} |
|
565 |
@{ML_antiquotation_def attributes} & : & @{text ML_antiquotation} \\ |
|
566 |
\end{matharray} |
|
567 |
||
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
51717
diff
changeset
|
568 |
@{rail \<open> |
45592 | 569 |
@@{ML_antiquotation attributes} attributes |
55112
b1a5d603fd12
prefer rail cartouche -- avoid back-slashed quotes;
wenzelm
parents:
51717
diff
changeset
|
570 |
\<close>} |
45592 | 571 |
|
572 |
\begin{description} |
|
573 |
||
574 |
\item @{text "@{attributes [\<dots>]}"} embeds attribute source |
|
575 |
representation into the ML text, which is particularly useful with |
|
576 |
declarations like @{ML Local_Theory.note}. Attribute names are |
|
577 |
internalized at compile time, but the source is unevaluated. This |
|
578 |
means attributes with formal arguments (types, terms, theorems) may |
|
579 |
be subject to odd effects of dynamic scoping! |
|
580 |
||
581 |
\end{description} |
|
582 |
*} |
|
583 |
||
39849 | 584 |
text %mlex {* See also @{command attribute_setup} in |
585 |
\cite{isabelle-isar-ref} which includes some abstract examples. *} |
|
30272 | 586 |
|
20472 | 587 |
end |