2
+ − 1
theory FirstSteps
25
+ − 2
imports Base
2
+ − 3
begin
+ − 4
+ − 5
chapter {* First Steps *}
+ − 6
42
+ − 7
text {*
+ − 8
54
+ − 9
Isabelle programming is done in ML. Just like lemmas and proofs, ML-code
89
+ − 10
in Isabelle is part of a theory. If you want to follow the code given in
54
+ − 11
this chapter, we assume you are working inside the theory starting with
2
+ − 12
6
+ − 13
\begin{center}
5
+ − 14
\begin{tabular}{@ {}l}
39
631d12c25bde
substantial changes to the antiquotations (preliminary version)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 15
\isacommand{theory} FirstSteps\\
5
+ − 16
\isacommand{imports} Main\\
+ − 17
\isacommand{begin}\\
6
+ − 18
\ldots
5
+ − 19
\end{tabular}
6
+ − 20
\end{center}
157
+ − 21
+ − 22
We also generally assume you are working with HOL. The given examples might
+ − 23
need to be adapted slightly if you work in a different logic.
14
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 24
*}
5
+ − 25
20
+ − 26
section {* Including ML-Code *}
14
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 27
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 28
text {*
5
+ − 29
The easiest and quickest way to include code in a theory is
89
+ − 30
by using the \isacommand{ML}-command. For example:
2
+ − 31
75
+ − 32
\begin{isabelle}
+ − 33
\begin{graybox}
85
+ − 34
\isacommand{ML}~@{text "\<verbopen>"}\isanewline
39
631d12c25bde
substantial changes to the antiquotations (preliminary version)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 35
\hspace{5mm}@{ML "3 + 4"}\isanewline
85
+ − 36
@{text "\<verbclose>"}\isanewline
+ − 37
@{text "> 7"}\smallskip
75
+ − 38
\end{graybox}
+ − 39
\end{isabelle}
2
+ − 40
102
5e309df58557
general cleaning up; deleted antiquotation ML_text; adjusted pathnames of various files in the distribution
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 41
Like normal Isabelle proof scripts, \isacommand{ML}-commands can be
5e309df58557
general cleaning up; deleted antiquotation ML_text; adjusted pathnames of various files in the distribution
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 42
evaluated by using the advance and undo buttons of your Isabelle
5e309df58557
general cleaning up; deleted antiquotation ML_text; adjusted pathnames of various files in the distribution
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 43
environment. The code inside the \isacommand{ML}-command can also contain
5e309df58557
general cleaning up; deleted antiquotation ML_text; adjusted pathnames of various files in the distribution
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 44
value and function bindings, and even those can be undone when the proof
160
cc9359bfacf4
redefined the functions warning and tracing in order to properly match more antiquotations
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 45
script is retracted. As mentioned in the Introduction, we will drop the
102
5e309df58557
general cleaning up; deleted antiquotation ML_text; adjusted pathnames of various files in the distribution
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 46
\isacommand{ML}~@{text "\<verbopen> \<dots> \<verbclose>"} scaffolding whenever we
107
+ − 47
show code. The lines prefixed with @{text [quotes] ">"} are not part of the
102
5e309df58557
general cleaning up; deleted antiquotation ML_text; adjusted pathnames of various files in the distribution
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 48
code, rather they indicate what the response is when the code is evaluated.
10
+ − 49
102
5e309df58557
general cleaning up; deleted antiquotation ML_text; adjusted pathnames of various files in the distribution
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 50
Once a portion of code is relatively stable, you usually want to export it
5e309df58557
general cleaning up; deleted antiquotation ML_text; adjusted pathnames of various files in the distribution
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 51
to a separate ML-file. Such files can then be included in a theory by using
5e309df58557
general cleaning up; deleted antiquotation ML_text; adjusted pathnames of various files in the distribution
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 52
the \isacommand{uses}-command in the header of the theory, like:
14
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 53
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 54
\begin{center}
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 55
\begin{tabular}{@ {}l}
54
+ − 56
\isacommand{theory} FirstSteps\\
14
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 57
\isacommand{imports} Main\\
58
+ − 58
\isacommand{uses} @{text "\"file_to_be_included.ML\""} @{text "\<dots>"}\\
14
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 59
\isacommand{begin}\\
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 60
\ldots
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 61
\end{tabular}
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 62
\end{center}
39
631d12c25bde
substantial changes to the antiquotations (preliminary version)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 63
14
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 64
*}
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 65
126
+ − 66
section {* Debugging and Printing\label{sec:printing} *}
14
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 67
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 68
text {*
13
+ − 69
50
+ − 70
During development you might find it necessary to inspect some data
10
+ − 71
in your code. This can be done in a ``quick-and-dirty'' fashion using
12
+ − 72
the function @{ML "warning"}. For example
10
+ − 73
161
+ − 74
@{ML_response_fake [display,gray] "warning \"any string\"" "\"any string\""}
10
+ − 75
58
+ − 76
will print out @{text [quotes] "any string"} inside the response buffer
+ − 77
of Isabelle. This function expects a string as argument. If you develop under PolyML,
50
+ − 78
then there is a convenient, though again ``quick-and-dirty'', method for
107
+ − 79
converting values into strings, namely the function @{ML makestring}:
10
+ − 80
161
+ − 81
@{ML_response_fake [display,gray] "warning (makestring 1)" "\"1\""}
12
+ − 82
196
+ − 83
However, @{ML makestring} only works if the type of what is converted is monomorphic
78
+ − 84
and not a function.
12
+ − 85
52
+ − 86
The function @{ML "warning"} should only be used for testing purposes, because any
+ − 87
output this function generates will be overwritten as soon as an error is
50
+ − 88
raised. For printing anything more serious and elaborate, the
54
+ − 89
function @{ML tracing} is more appropriate. This function writes all output into
89
+ − 90
a separate tracing buffer. For example:
14
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 91
161
+ − 92
@{ML_response_fake [display,gray] "tracing \"foo\"" "\"foo\""}
14
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 93
58
+ − 94
It is also possible to redirect the ``channel'' where the string @{text "foo"} is
196
+ − 95
printed to a separate file, e.g., to prevent ProofGeneral from choking on massive
107
+ − 96
amounts of trace output. This redirection can be achieved with the code:
43
02f76f1b6e7b
added positions to anti-quotations; removed old antiquotation_setup; tuned the text a bit
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 97
*}
14
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 98
69
+ − 99
ML{*val strip_specials =
42
+ − 100
let
43
02f76f1b6e7b
added positions to anti-quotations; removed old antiquotation_setup; tuned the text a bit
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 101
fun strip ("\^A" :: _ :: cs) = strip cs
42
+ − 102
| strip (c :: cs) = c :: strip cs
+ − 103
| strip [] = [];
+ − 104
in implode o strip o explode end;
+ − 105
+ − 106
fun redirect_tracing stream =
+ − 107
Output.tracing_fn := (fn s =>
14
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 108
(TextIO.output (stream, (strip_specials s));
43
02f76f1b6e7b
added positions to anti-quotations; removed old antiquotation_setup; tuned the text a bit
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 109
TextIO.output (stream, "\n");
69
+ − 110
TextIO.flushOut stream)) *}
14
1c17e99f6f66
added a paragraph about "uses" and started a paragraph about tracing
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 111
43
02f76f1b6e7b
added positions to anti-quotations; removed old antiquotation_setup; tuned the text a bit
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 112
text {*
02f76f1b6e7b
added positions to anti-quotations; removed old antiquotation_setup; tuned the text a bit
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 113
Calling @{ML "redirect_tracing"} with @{ML "(TextIO.openOut \"foo.bar\")"}
58
+ − 114
will cause that all tracing information is printed into the file @{text "foo.bar"}.
75
+ − 115
107
+ − 116
You can print out error messages with the function @{ML error}; for example:
75
+ − 117
122
+ − 118
@{ML_response_fake [display,gray] "if 0=1 then true else (error \"foo\")"
+ − 119
"Exception- ERROR \"foo\" raised
+ − 120
At command \"ML\"."}
75
+ − 121
192
+ − 122
(FIXME @{ML Toplevel.debug} @{ML Toplevel.profiling})
+ − 123
*}
+ − 124
+ − 125
(*
+ − 126
ML {*
+ − 127
fun dodgy_fun () = (raise (ERROR "bar"); 1)
+ − 128
*}
+ − 129
+ − 130
ML {* set Toplevel.debug *}
+ − 131
+ − 132
ML {* fun f1 () = dodgy_fun () *}
+ − 133
+ − 134
ML {* f1 () *}
+ − 135
*)
+ − 136
+ − 137
text {*
126
+ − 138
Most often you want to inspect data of type @{ML_type term}, @{ML_type cterm}
+ − 139
or @{ML_type thm}. Isabelle contains elaborate pretty-printing functions for printing them,
+ − 140
but for quick-and-dirty solutions they are far too unwieldy. A simple way to transform
+ − 141
a term into a string is to use the function @{ML Syntax.string_of_term}.
+ − 142
+ − 143
@{ML_response_fake [display,gray]
+ − 144
"Syntax.string_of_term @{context} @{term \"1::nat\"}"
+ − 145
"\"\\^E\\^Fterm\\^E\\^E\\^Fconst\\^Fname=HOL.one_class.one\\^E1\\^E\\^F\\^E\\^E\\^F\\^E\""}
+ − 146
+ − 147
This produces a string with some additional information encoded in it. The string
+ − 148
can be properly printed by using the function @{ML warning}.
+ − 149
+ − 150
@{ML_response_fake [display,gray]
+ − 151
"warning (Syntax.string_of_term @{context} @{term \"1::nat\"})"
+ − 152
"\"1\""}
+ − 153
+ − 154
A @{ML_type cterm} can be transformed into a string by the following function.
+ − 155
*}
+ − 156
+ − 157
ML{*fun str_of_cterm ctxt t =
+ − 158
Syntax.string_of_term ctxt (term_of t)*}
+ − 159
+ − 160
text {*
149
+ − 161
In this example the function @{ML term_of} extracts the @{ML_type term} from
+ − 162
a @{ML_type cterm}. If there are more than one @{ML_type cterm}s to be
+ − 163
printed, you can use the function @{ML commas} to separate them.
126
+ − 164
*}
+ − 165
+ − 166
ML{*fun str_of_cterms ctxt ts =
+ − 167
commas (map (str_of_cterm ctxt) ts)*}
+ − 168
+ − 169
text {*
+ − 170
The easiest way to get the string of a theorem is to transform it
190
+ − 171
into a @{ML_type cterm} using the function @{ML crep_thm}.
+ − 172
*}
+ − 173
+ − 174
ML{*fun str_of_thm_raw ctxt thm =
+ − 175
str_of_cterm ctxt (#prop (crep_thm thm))*}
+ − 176
+ − 177
text {*
+ − 178
Theorems also include schematic variables, such as @{text "?P"},
+ − 179
@{text "?Q"} and so on.
+ − 180
+ − 181
@{ML_response_fake [display, gray]
+ − 182
"warning (str_of_thm_raw @{context} @{thm conjI})"
+ − 183
"\<lbrakk>?P; ?Q\<rbrakk> \<Longrightarrow> ?P \<and> ?Q"}
+ − 184
+ − 185
In order to improve the readability of theorems we convert
158
d7944bdf7b3f
removed infix_conv and moved function no_vars into the FirstSteps chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 186
these schematic variables into free variables using the
d7944bdf7b3f
removed infix_conv and moved function no_vars into the FirstSteps chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 187
function @{ML Variable.import_thms}.
126
+ − 188
*}
+ − 189
158
d7944bdf7b3f
removed infix_conv and moved function no_vars into the FirstSteps chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 190
ML{*fun no_vars ctxt thm =
d7944bdf7b3f
removed infix_conv and moved function no_vars into the FirstSteps chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 191
let
d7944bdf7b3f
removed infix_conv and moved function no_vars into the FirstSteps chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 192
val ((_, [thm']), _) = Variable.import_thms true [thm] ctxt
d7944bdf7b3f
removed infix_conv and moved function no_vars into the FirstSteps chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 193
in
d7944bdf7b3f
removed infix_conv and moved function no_vars into the FirstSteps chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 194
thm'
d7944bdf7b3f
removed infix_conv and moved function no_vars into the FirstSteps chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 195
end
d7944bdf7b3f
removed infix_conv and moved function no_vars into the FirstSteps chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 196
d7944bdf7b3f
removed infix_conv and moved function no_vars into the FirstSteps chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 197
fun str_of_thm ctxt thm =
171
+ − 198
str_of_cterm ctxt (#prop (crep_thm (no_vars ctxt thm)))*}
126
+ − 199
+ − 200
text {*
190
+ − 201
Theorem @{thm [source] conjI} looks now as follows
+ − 202
+ − 203
@{ML_response_fake [display, gray]
196
+ − 204
"warning (str_of_thm @{context} @{thm conjI})"
+ − 205
"\<lbrakk>P; Q\<rbrakk> \<Longrightarrow> P \<and> Q"}
190
+ − 206
126
+ − 207
Again the function @{ML commas} helps with printing more than one theorem.
+ − 208
*}
+ − 209
+ − 210
ML{*fun str_of_thms ctxt thms =
190
+ − 211
commas (map (str_of_thm ctxt) thms)
+ − 212
+ − 213
fun str_of_thms_raw ctxt thms =
+ − 214
commas (map (str_of_thm_raw ctxt) thms)*}
126
+ − 215
+ − 216
section {* Combinators\label{sec:combinators} *}
+ − 217
+ − 218
text {*
131
+ − 219
For beginners perhaps the most puzzling parts in the existing code of Isabelle are
126
+ − 220
the combinators. At first they seem to greatly obstruct the
+ − 221
comprehension of the code, but after getting familiar with them, they
+ − 222
actually ease the understanding and also the programming.
+ − 223
+ − 224
The simplest combinator is @{ML I}, which is just the identity function defined as
+ − 225
*}
+ − 226
+ − 227
ML{*fun I x = x*}
+ − 228
+ − 229
text {* Another simple combinator is @{ML K}, defined as *}
+ − 230
+ − 231
ML{*fun K x = fn _ => x*}
+ − 232
+ − 233
text {*
+ − 234
@{ML K} ``wraps'' a function around the argument @{text "x"}. However, this
+ − 235
function ignores its argument. As a result, @{ML K} defines a constant function
+ − 236
always returning @{text x}.
+ − 237
+ − 238
The next combinator is reverse application, @{ML "|>"}, defined as:
+ − 239
*}
+ − 240
+ − 241
ML{*fun x |> f = f x*}
+ − 242
+ − 243
text {* While just syntactic sugar for the usual function application,
+ − 244
the purpose of this combinator is to implement functions in a
+ − 245
``waterfall fashion''. Consider for example the function *}
+ − 246
+ − 247
ML %linenosgray{*fun inc_by_five x =
+ − 248
x |> (fn x => x + 1)
+ − 249
|> (fn x => (x, x))
+ − 250
|> fst
+ − 251
|> (fn x => x + 4)*}
+ − 252
+ − 253
text {*
196
+ − 254
which increments its argument @{text x} by 5. It proceeds by first incrementing
126
+ − 255
the argument by 1 (Line 2); then storing the result in a pair (Line 3); taking
+ − 256
the first component of the pair (Line 4) and finally incrementing the first
+ − 257
component by 4 (Line 5). This kind of cascading manipulations of values is quite
+ − 258
common when dealing with theories (for example by adding a definition, followed by
+ − 259
lemmas and so on). The reverse application allows you to read what happens in
+ − 260
a top-down manner. This kind of coding should also be familiar,
149
+ − 261
if you have been exposed to Haskell's do-notation. Writing the function @{ML inc_by_five} using
126
+ − 262
the reverse application is much clearer than writing
+ − 263
*}
+ − 264
+ − 265
ML{*fun inc_by_five x = fst ((fn x => (x, x)) (x + 1)) + 4*}
+ − 266
+ − 267
text {* or *}
+ − 268
+ − 269
ML{*fun inc_by_five x =
+ − 270
((fn x => x + 4) o fst o (fn x => (x, x)) o (fn x => x + 1)) x*}
+ − 271
+ − 272
text {* and typographically more economical than *}
+ − 273
+ − 274
ML{*fun inc_by_five x =
+ − 275
let val y1 = x + 1
+ − 276
val y2 = (y1, y1)
+ − 277
val y3 = fst y2
+ − 278
val y4 = y3 + 4
+ − 279
in y4 end*}
+ − 280
+ − 281
text {*
+ − 282
Another reason why the let-bindings in the code above are better to be
+ − 283
avoided: it is more than easy to get the intermediate values wrong, not to
+ − 284
mention the nightmares the maintenance of this code causes!
+ − 285
178
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 286
In the context of Isabelle, a ``real world'' example for a function written in
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 287
the waterfall fashion might be the following code:
177
+ − 288
*}
126
+ − 289
177
+ − 290
ML %linenosgray{*fun apply_fresh_args pred ctxt =
+ − 291
pred |> fastype_of
+ − 292
|> binder_types
+ − 293
|> map (pair "z")
+ − 294
|> Variable.variant_frees ctxt [pred]
+ − 295
|> map Free
+ − 296
|> (curry list_comb) pred *}
126
+ − 297
177
+ − 298
text {*
184
+ − 299
This code extracts the argument types of a given
+ − 300
predicate and then generates for each argument type a distinct variable; finally it
183
+ − 301
applies the generated variables to the predicate. For example
+ − 302
+ − 303
@{ML_response_fake [display,gray]
+ − 304
"apply_fresh_args @{term \"P::nat \<Rightarrow> int \<Rightarrow> unit \<Rightarrow> bool\"} @{context}
+ − 305
|> Syntax.string_of_term @{context}
+ − 306
|> warning"
+ − 307
"P z za zb"}
177
+ − 308
184
+ − 309
You can read off this behaviour from how @{ML apply_fresh_args} is
183
+ − 310
coded: in Line 2, the function @{ML fastype_of} calculates the type of the
184
+ − 311
predicate; @{ML binder_types} in the next line produces the list of argument
+ − 312
types (in the case above the list @{text "[nat, int, unit]"}); Line 4
+ − 313
pairs up each type with the string @{text "z"}; the
183
+ − 314
function @{ML variant_frees in Variable} generates for each @{text "z"} a
184
+ − 315
unique name avoiding the given @{text pred}; the list of name-type pairs is turned
+ − 316
into a list of variable terms in Line 6, which in the last line is applied
183
+ − 317
by the function @{ML list_comb} to the predicate. We have to use the
+ − 318
function @{ML curry}, because @{ML list_comb} expects the predicate and the
184
+ − 319
variables list as a pair.
177
+ − 320
+ − 321
The combinator @{ML "#>"} is the reverse function composition. It can be
+ − 322
used to define the following function
126
+ − 323
*}
+ − 324
+ − 325
ML{*val inc_by_six =
+ − 326
(fn x => x + 1)
+ − 327
#> (fn x => x + 2)
+ − 328
#> (fn x => x + 3)*}
+ − 329
+ − 330
text {*
+ − 331
which is the function composed of first the increment-by-one function and then
+ − 332
increment-by-two, followed by increment-by-three. Again, the reverse function
+ − 333
composition allows you to read the code top-down.
+ − 334
+ − 335
The remaining combinators described in this section add convenience for the
+ − 336
``waterfall method'' of writing functions. The combinator @{ML tap} allows
+ − 337
you to get hold of an intermediate result (to do some side-calculations for
+ − 338
instance). The function
+ − 339
+ − 340
*}
+ − 341
+ − 342
ML %linenosgray{*fun inc_by_three x =
+ − 343
x |> (fn x => x + 1)
+ − 344
|> tap (fn x => tracing (makestring x))
+ − 345
|> (fn x => x + 2)*}
+ − 346
+ − 347
text {*
+ − 348
increments the argument first by @{text "1"} and then by @{text "2"}. In the
+ − 349
middle (Line 3), however, it uses @{ML tap} for printing the ``plus-one''
+ − 350
intermediate result inside the tracing buffer. The function @{ML tap} can
+ − 351
only be used for side-calculations, because any value that is computed
+ − 352
cannot be merged back into the ``main waterfall''. To do this, you can use
+ − 353
the next combinator.
+ − 354
196
+ − 355
The combinator @{ML "`"} (a backtick) is similar to @{ML tap}, but applies a
+ − 356
function to the value and returns the result together with the value (as a
+ − 357
pair). For example the function
126
+ − 358
*}
+ − 359
+ − 360
ML{*fun inc_as_pair x =
+ − 361
x |> `(fn x => x + 1)
+ − 362
|> (fn (x, y) => (x, y + 1))*}
+ − 363
+ − 364
text {*
+ − 365
takes @{text x} as argument, and then increments @{text x}, but also keeps
+ − 366
@{text x}. The intermediate result is therefore the pair @{ML "(x + 1, x)"
+ − 367
for x}. After that, the function increments the right-hand component of the
+ − 368
pair. So finally the result will be @{ML "(x + 1, x + 1)" for x}.
+ − 369
+ − 370
The combinators @{ML "|>>"} and @{ML "||>"} are defined for
+ − 371
functions manipulating pairs. The first applies the function to
+ − 372
the first component of the pair, defined as
+ − 373
*}
+ − 374
+ − 375
ML{*fun (x, y) |>> f = (f x, y)*}
+ − 376
+ − 377
text {*
+ − 378
and the second combinator to the second component, defined as
+ − 379
*}
+ − 380
+ − 381
ML{*fun (x, y) ||> f = (x, f y)*}
+ − 382
+ − 383
text {*
+ − 384
With the combinator @{ML "|->"} you can re-combine the elements from a pair.
+ − 385
This combinator is defined as
+ − 386
*}
+ − 387
+ − 388
ML{*fun (x, y) |-> f = f x y*}
+ − 389
+ − 390
text {* and can be used to write the following roundabout version
+ − 391
of the @{text double} function:
+ − 392
*}
+ − 393
+ − 394
ML{*fun double x =
+ − 395
x |> (fn x => (x, x))
+ − 396
|-> (fn x => fn y => x + y)*}
+ − 397
+ − 398
text {*
196
+ − 399
Recall that @{ML "|>"} is the reverse function application. Recall also that
+ − 400
the related
126
+ − 401
reverse function composition is @{ML "#>"}. In fact all the combinators @{ML "|->"},
+ − 402
@{ML "|>>"} and @{ML "||>"} described above have related combinators for function
+ − 403
composition, namely @{ML "#->"}, @{ML "#>>"} and @{ML "##>"}. Using @{ML "#->"},
+ − 404
for example, the function @{text double} can also be written as:
+ − 405
*}
+ − 406
+ − 407
ML{*val double =
+ − 408
(fn x => (x, x))
+ − 409
#-> (fn x => fn y => x + y)*}
+ − 410
+ − 411
text {*
+ − 412
+ − 413
(FIXME: find a good exercise for combinators)
127
+ − 414
+ − 415
\begin{readmore}
196
+ − 416
The most frequently used combinators are defined in the files @{ML_file
+ − 417
"Pure/library.ML"}
127
+ − 418
and @{ML_file "Pure/General/basics.ML"}. Also \isccite{sec:ML-linear-trans}
+ − 419
contains further information about combinators.
+ − 420
\end{readmore}
126
+ − 421
15
+ − 422
*}
+ − 423
10
+ − 424
2
+ − 425
section {* Antiquotations *}
+ − 426
+ − 427
text {*
49
+ − 428
The main advantage of embedding all code in a theory is that the code can
58
+ − 429
contain references to entities defined on the logical level of Isabelle. By
+ − 430
this we mean definitions, theorems, terms and so on. This kind of reference is
+ − 431
realised with antiquotations. For example, one can print out the name of the current
49
+ − 432
theory by typing
+ − 433
39
631d12c25bde
substantial changes to the antiquotations (preliminary version)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 434
72
7b8c4fe235aa
added an antiquotation option [gray] for gray boxes around displays
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 435
@{ML_response [display,gray] "Context.theory_name @{theory}" "\"FirstSteps\""}
39
631d12c25bde
substantial changes to the antiquotations (preliminary version)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 436
5
+ − 437
where @{text "@{theory}"} is an antiquotation that is substituted with the
49
+ − 438
current theory (remember that we assumed we are inside the theory
89
+ − 439
@{text FirstSteps}). The name of this theory can be extracted using
49
+ − 440
the function @{ML "Context.theory_name"}.
5
+ − 441
89
+ − 442
Note, however, that antiquotations are statically linked, that is their value is
12
+ − 443
determined at ``compile-time'', not ``run-time''. For example the function
43
02f76f1b6e7b
added positions to anti-quotations; removed old antiquotation_setup; tuned the text a bit
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 444
*}
5
+ − 445
69
+ − 446
ML{*fun not_current_thyname () = Context.theory_name @{theory} *}
43
02f76f1b6e7b
added positions to anti-quotations; removed old antiquotation_setup; tuned the text a bit
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 447
02f76f1b6e7b
added positions to anti-quotations; removed old antiquotation_setup; tuned the text a bit
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 448
text {*
2
+ − 449
89
+ − 450
does \emph{not} return the name of the current theory, if it is run in a
5
+ − 451
different theory. Instead, the code above defines the constant function
58
+ − 452
that always returns the string @{text [quotes] "FirstSteps"}, no matter where the
43
02f76f1b6e7b
added positions to anti-quotations; removed old antiquotation_setup; tuned the text a bit
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 453
function is called. Operationally speaking, the antiquotation @{text "@{theory}"} is
5
+ − 454
\emph{not} replaced with code that will look up the current theory in
+ − 455
some data structure and return it. Instead, it is literally
+ − 456
replaced with the value representing the theory name.
2
+ − 457
132
+ − 458
In a similar way you can use antiquotations to refer to proved theorems:
133
+ − 459
@{text "@{thm \<dots>}"} for a single theorem
39
631d12c25bde
substantial changes to the antiquotations (preliminary version)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 460
72
7b8c4fe235aa
added an antiquotation option [gray] for gray boxes around displays
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 461
@{ML_response_fake [display,gray] "@{thm allI}" "(\<And>x. ?P x) \<Longrightarrow> \<forall>x. ?P x"}
75
+ − 462
133
+ − 463
and @{text "@{thms \<dots>}"} for more than one
132
+ − 464
+ − 465
@{ML_response_fake [display,gray] "@{thms conj_ac}"
+ − 466
"(?P \<and> ?Q) = (?Q \<and> ?P)
+ − 467
(?P \<and> ?Q \<and> ?R) = (?Q \<and> ?P \<and> ?R)
+ − 468
((?P \<and> ?Q) \<and> ?R) = (?P \<and> ?Q \<and> ?R)"}
+ − 469
149
+ − 470
You can also refer to the current simpset. To illustrate this we implement the
132
+ − 471
function that extracts the theorem names stored in a simpset.
131
+ − 472
*}
75
+ − 473
149
+ − 474
ML{*fun get_thm_names_from_ss simpset =
131
+ − 475
let
163
2319cff107f0
removed rep_ss, and used dest_ss instead; some very slight changes to simple_inductive
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 476
val {simps,...} = MetaSimplifier.dest_ss simpset
70
+ − 477
in
163
2319cff107f0
removed rep_ss, and used dest_ss instead; some very slight changes to simple_inductive
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 478
map #1 simps
131
+ − 479
end*}
54
+ − 480
131
+ − 481
text {*
163
2319cff107f0
removed rep_ss, and used dest_ss instead; some very slight changes to simple_inductive
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 482
The function @{ML dest_ss in MetaSimplifier} returns a record containing all
184
+ − 483
information stored in the simpset. We are only interested in the names of the
+ − 484
simp-rules. So now you can feed in the current simpset into this function.
+ − 485
The simpset can be referred to using the antiquotation @{text "@{simpset}"}.
81
+ − 486
131
+ − 487
@{ML_response_fake [display,gray]
149
+ − 488
"get_thm_names_from_ss @{simpset}"
+ − 489
"[\"Nat.of_nat_eq_id\", \"Int.of_int_eq_id\", \"Nat.One_nat_def\", \<dots>]"}
10
+ − 490
196
+ − 491
Again, this way of referencing simpsets makes you independent from additions
156
+ − 492
of lemmas to the simpset by the user that potentially cause loops.
+ − 493
192
+ − 494
On the ML-level of Isabelle, you often have to work with qualified names;
196
+ − 495
these are strings with some additional information, such as positional information
192
+ − 496
and qualifiers. Such bindings can be generated with the antiquotation
196
+ − 497
@{text "@{binding \<dots>}"}.
192
+ − 498
+ − 499
@{ML_response [display,gray]
+ − 500
"@{binding \"name\"}"
+ − 501
"name"}
+ − 502
196
+ − 503
An example where a binding is needed is the function @{ML define in
+ − 504
LocalTheory}. Below, this function is used to define the constant @{term
+ − 505
"TrueConj"} as the conjunction
192
+ − 506
@{term "True \<and> True"}.
+ − 507
*}
+ − 508
+ − 509
local_setup %gray {*
+ − 510
snd o LocalTheory.define Thm.internalK
+ − 511
((@{binding "TrueConj"}, NoSyn),
+ − 512
(Attrib.empty_binding, @{term "True \<and> True"})) *}
+ − 513
+ − 514
text {*
196
+ − 515
While antiquotations have many applications, they were originally introduced
+ − 516
in order to avoid explicit bindings of theorems such as:
43
02f76f1b6e7b
added positions to anti-quotations; removed old antiquotation_setup; tuned the text a bit
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 517
*}
02f76f1b6e7b
added positions to anti-quotations; removed old antiquotation_setup; tuned the text a bit
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 518
69
+ − 519
ML{*val allI = thm "allI" *}
43
02f76f1b6e7b
added positions to anti-quotations; removed old antiquotation_setup; tuned the text a bit
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 520
02f76f1b6e7b
added positions to anti-quotations; removed old antiquotation_setup; tuned the text a bit
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 521
text {*
196
+ − 522
Such bindings are difficult to maintain and can be overwritten by the
+ − 523
user accidentally. This often broke Isabelle
49
+ − 524
packages. Antiquotations solve this problem, since they are ``linked''
89
+ − 525
statically at compile-time. However, this static linkage also limits their
+ − 526
usefulness in cases where data needs to be build up dynamically. In the
196
+ − 527
course of this chapter you will learn more about antiquotations:
122
+ − 528
they can simplify Isabelle programming since one can directly access all
196
+ − 529
kinds of logical elements from the ML-level.
2
+ − 530
*}
+ − 531
15
+ − 532
section {* Terms and Types *}
2
+ − 533
+ − 534
text {*
122
+ − 535
One way to construct terms of Isabelle is by using the antiquotation
89
+ − 536
\mbox{@{text "@{term \<dots>}"}}. For example:
2
+ − 537
72
7b8c4fe235aa
added an antiquotation option [gray] for gray boxes around displays
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 538
@{ML_response [display,gray]
75
+ − 539
"@{term \"(a::nat) + b = c\"}"
+ − 540
"Const (\"op =\", \<dots>) $
149
+ − 541
(Const (\"HOL.plus_class.plus\", \<dots>) $ \<dots> $ \<dots>) $ \<dots>"}
2
+ − 542
50
+ − 543
This will show the term @{term "(a::nat) + b = c"}, but printed using the internal
13
+ − 544
representation of this term. This internal representation corresponds to the
39
631d12c25bde
substantial changes to the antiquotations (preliminary version)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 545
datatype @{ML_type "term"}.
2
+ − 546
34
+ − 547
The internal representation of terms uses the usual de Bruijn index mechanism where bound
11
+ − 548
variables are represented by the constructor @{ML Bound}. The index in @{ML Bound} refers to
10
+ − 549
the number of Abstractions (@{ML Abs}) we have to skip until we hit the @{ML Abs} that
12
+ − 550
binds the corresponding variable. However, in Isabelle the names of bound variables are
149
+ − 551
kept at abstractions for printing purposes, and so should be treated only as ``comments''.
123
+ − 552
Application in Isabelle is realised with the term-constructor @{ML $}.
10
+ − 553
2
+ − 554
\begin{readmore}
13
+ − 555
Terms are described in detail in \isccite{sec:terms}. Their
78
+ − 556
definition and many useful operations are implemented in @{ML_file "Pure/term.ML"}.
2
+ − 557
\end{readmore}
+ − 558
13
+ − 559
Sometimes the internal representation of terms can be surprisingly different
157
+ − 560
from what you see at the user-level, because the layers of
47
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 561
parsing/type-checking/pretty printing can be quite elaborate.
2
+ − 562
10
+ − 563
\begin{exercise}
2
+ − 564
Look at the internal term representation of the following terms, and
89
+ − 565
find out why they are represented like this:
2
+ − 566
+ − 567
\begin{itemize}
+ − 568
\item @{term "case x of 0 \<Rightarrow> 0 | Suc y \<Rightarrow> y"}
+ − 569
\item @{term "\<lambda>(x,y). P y x"}
+ − 570
\item @{term "{ [x::int] | x. x \<le> -2 }"}
+ − 571
\end{itemize}
+ − 572
+ − 573
Hint: The third term is already quite big, and the pretty printer
+ − 574
may omit parts of it by default. If you want to see all of it, you
122
+ − 575
can use the following ML-function to set the printing depth to a higher
+ − 576
value:
12
+ − 577
75
+ − 578
@{ML [display,gray] "print_depth 50"}
72
7b8c4fe235aa
added an antiquotation option [gray] for gray boxes around displays
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 579
\end{exercise}
39
631d12c25bde
substantial changes to the antiquotations (preliminary version)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 580
13
+ − 581
The antiquotation @{text "@{prop \<dots>}"} constructs terms of propositional type,
50
+ − 582
inserting the invisible @{text "Trueprop"}-coercions whenever necessary.
68
+ − 583
Consider for example the pairs
12
+ − 584
126
+ − 585
@{ML_response [display,gray] "(@{term \"P x\"}, @{prop \"P x\"})"
+ − 586
"(Free (\"P\", \<dots>) $ Free (\"x\", \<dots>),
149
+ − 587
Const (\"Trueprop\", \<dots>) $ (Free (\"P\", \<dots>) $ Free (\"x\", \<dots>)))"}
65
+ − 588
108
8bea3f74889d
added to the tactical chapter; polished; added the tabularstar environment (which is just tabular*)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 589
where a coercion is inserted in the second component and
12
+ − 590
72
7b8c4fe235aa
added an antiquotation option [gray] for gray boxes around displays
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 591
@{ML_response [display,gray] "(@{term \"P x \<Longrightarrow> Q x\"}, @{prop \"P x \<Longrightarrow> Q x\"})"
65
+ − 592
"(Const (\"==>\", \<dots>) $ \<dots> $ \<dots>, Const (\"==>\", \<dots>) $ \<dots> $ \<dots>)"}
12
+ − 593
72
7b8c4fe235aa
added an antiquotation option [gray] for gray boxes around displays
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 594
where it is not (since it is already constructed by a meta-implication).
19
+ − 595
89
+ − 596
Types can be constructed using the antiquotation @{text "@{typ \<dots>}"}. For example:
39
631d12c25bde
substantial changes to the antiquotations (preliminary version)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 597
72
7b8c4fe235aa
added an antiquotation option [gray] for gray boxes around displays
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 598
@{ML_response_fake [display,gray] "@{typ \"bool \<Rightarrow> nat\"}" "bool \<Rightarrow> nat"}
39
631d12c25bde
substantial changes to the antiquotations (preliminary version)
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 599
19
+ − 600
\begin{readmore}
+ − 601
Types are described in detail in \isccite{sec:types}. Their
78
+ − 602
definition and many useful operations are implemented
+ − 603
in @{ML_file "Pure/type.ML"}.
19
+ − 604
\end{readmore}
47
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 605
*}
19
+ − 606
+ − 607
156
+ − 608
section {* Constructing Terms and Types Manually\label{sec:terms_types_manually} *}
12
+ − 609
+ − 610
text {*
81
+ − 611
While antiquotations are very convenient for constructing terms, they can
102
5e309df58557
general cleaning up; deleted antiquotation ML_text; adjusted pathnames of various files in the distribution
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 612
only construct fixed terms (remember they are ``linked'' at compile-time).
5e309df58557
general cleaning up; deleted antiquotation ML_text; adjusted pathnames of various files in the distribution
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 613
However, you often need to construct terms dynamically. For example, a
186
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 614
function that returns the implication @{text "\<And>(x::nat). P x \<Longrightarrow> Q x"} taking
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 615
@{term P} and @{term Q} as arguments can only be written as:
102
5e309df58557
general cleaning up; deleted antiquotation ML_text; adjusted pathnames of various files in the distribution
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 616
43
02f76f1b6e7b
added positions to anti-quotations; removed old antiquotation_setup; tuned the text a bit
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 617
*}
12
+ − 618
186
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 619
ML{*fun make_imp P Q =
131
+ − 620
let
186
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 621
val x = Free ("x", @{typ nat})
131
+ − 622
in
+ − 623
Logic.all x (Logic.mk_implies (P $ x, Q $ x))
+ − 624
end *}
43
02f76f1b6e7b
added positions to anti-quotations; removed old antiquotation_setup; tuned the text a bit
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 625
02f76f1b6e7b
added positions to anti-quotations; removed old antiquotation_setup; tuned the text a bit
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 626
text {*
186
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 627
The reason is that you cannot pass the arguments @{term P} and @{term Q}
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 628
into an antiquotation. For example the following does \emph{not} work.
43
02f76f1b6e7b
added positions to anti-quotations; removed old antiquotation_setup; tuned the text a bit
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 629
*}
13
+ − 630
186
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 631
ML{*fun make_wrong_imp P Q = @{prop "\<And>(x::nat). P x \<Longrightarrow> Q x"} *}
12
+ − 632
43
02f76f1b6e7b
added positions to anti-quotations; removed old antiquotation_setup; tuned the text a bit
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 633
text {*
186
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 634
To see this apply @{text "@{term S}"} and @{text "@{term T}"}
75
+ − 635
to both functions. With @{ML make_imp} we obtain the intended term involving
102
5e309df58557
general cleaning up; deleted antiquotation ML_text; adjusted pathnames of various files in the distribution
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 636
the given arguments
65
+ − 637
186
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 638
@{ML_response [display,gray] "make_imp @{term S} @{term T}"
162
+ − 639
"Const \<dots> $
+ − 640
Abs (\"x\", Type (\"nat\",[]),
+ − 641
Const \<dots> $ (Free (\"S\",\<dots>) $ \<dots>) $ (Free (\"T\",\<dots>) $ \<dots>))"}
68
+ − 642
81
+ − 643
whereas with @{ML make_wrong_imp} we obtain a term involving the @{term "P"}
68
+ − 644
and @{text "Q"} from the antiquotation.
+ − 645
186
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 646
@{ML_response [display,gray] "make_wrong_imp @{term S} @{term T}"
162
+ − 647
"Const \<dots> $
+ − 648
Abs (\"x\", \<dots>,
+ − 649
Const \<dots> $ (Const \<dots> $ (Free (\"P\",\<dots>) $ \<dots>)) $
192
+ − 650
(Const \<dots> $ (Free (\"Q\",\<dots>) $ \<dots>)))"}
65
+ − 651
192
+ − 652
There are a number of handy functions that are frequently used for
+ − 653
constructing terms. One is the function @{ML list_comb} which a term
+ − 654
and a list of terms as argument, and produces as output the term
+ − 655
list applied to the term. For example
+ − 656
+ − 657
@{ML_response_fake [display,gray]
+ − 658
"list_comb (@{term \"P::nat\"}, [@{term \"True\"}, @{term \"False\"}])"
+ − 659
"Free (\"P\", \"nat\") $ Const (\"True\", \"bool\") $ Const (\"False\", \"bool\")"}
+ − 660
+ − 661
(FIXME: handy functions for constructing terms: @{ML lambda},
190
+ − 662
@{ML subst_free})
186
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 663
*}
49
+ − 664
192
+ − 665
ML {* lambda @{term "x::nat"} @{term "P x"}*}
+ − 666
49
+ − 667
+ − 668
text {*
192
+ − 669
As can be seen this function does not take the typing annotation into account.
+ − 670
13
+ − 671
\begin{readmore}
89
+ − 672
There are many functions in @{ML_file "Pure/term.ML"}, @{ML_file "Pure/logic.ML"} and
102
5e309df58557
general cleaning up; deleted antiquotation ML_text; adjusted pathnames of various files in the distribution
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 673
@{ML_file "HOL/Tools/hologic.ML"} that make such manual constructions of terms
49
+ − 674
and types easier.\end{readmore}
13
+ − 675
+ − 676
Have a look at these files and try to solve the following two exercises:
11
+ − 677
*}
+ − 678
+ − 679
text {*
+ − 680
13
+ − 681
\begin{exercise}\label{fun:revsum}
58
+ − 682
Write a function @{text "rev_sum : term -> term"} that takes a
122
+ − 683
term of the form @{text "t\<^isub>1 + t\<^isub>2 + \<dots> + t\<^isub>n"} (whereby @{text "n"} might be zero)
11
+ − 684
and returns the reversed sum @{text "t\<^isub>n + \<dots> + t\<^isub>2 + t\<^isub>1"}. Assume
+ − 685
the @{text "t\<^isub>i"} can be arbitrary expressions and also note that @{text "+"}
13
+ − 686
associates to the left. Try your function on some examples.
11
+ − 687
\end{exercise}
+ − 688
15
+ − 689
\begin{exercise}\label{fun:makesum}
11
+ − 690
Write a function which takes two terms representing natural numbers
75
+ − 691
in unary notation (like @{term "Suc (Suc (Suc 0))"}), and produce the
11
+ − 692
number representing their sum.
+ − 693
\end{exercise}
+ − 694
122
+ − 695
There are a few subtle issues with constants. They usually crop up when
149
+ − 696
pattern matching terms or types, or when constructing them. While it is perfectly ok
122
+ − 697
to write the function @{text is_true} as follows
+ − 698
*}
+ − 699
+ − 700
ML{*fun is_true @{term True} = true
+ − 701
| is_true _ = false*}
+ − 702
+ − 703
text {*
+ − 704
this does not work for picking out @{text "\<forall>"}-quantified terms. Because
+ − 705
the function
+ − 706
*}
+ − 707
+ − 708
ML{*fun is_all (@{term All} $ _) = true
+ − 709
| is_all _ = false*}
+ − 710
+ − 711
text {*
123
+ − 712
will not correctly match the formula @{prop "\<forall>x::nat. P x"}:
122
+ − 713
+ − 714
@{ML_response [display,gray] "is_all @{term \"\<forall>x::nat. P x\"}" "false"}
+ − 715
+ − 716
The problem is that the @{text "@term"}-antiquotation in the pattern
123
+ − 717
fixes the type of the constant @{term "All"} to be @{typ "('a \<Rightarrow> bool) \<Rightarrow> bool"} for
122
+ − 718
an arbitrary, but fixed type @{typ "'a"}. A properly working alternative
+ − 719
for this function is
+ − 720
*}
+ − 721
+ − 722
ML{*fun is_all (Const ("All", _) $ _) = true
+ − 723
| is_all _ = false*}
+ − 724
+ − 725
text {*
+ − 726
because now
+ − 727
+ − 728
@{ML_response [display,gray] "is_all @{term \"\<forall>x::nat. P x\"}" "true"}
+ − 729
149
+ − 730
matches correctly (the first wildcard in the pattern matches any type and the
+ − 731
second any term).
122
+ − 732
123
+ − 733
However there is still a problem: consider the similar function that
131
+ − 734
attempts to pick out @{text "Nil"}-terms:
122
+ − 735
*}
+ − 736
+ − 737
ML{*fun is_nil (Const ("Nil", _)) = true
+ − 738
| is_nil _ = false *}
+ − 739
+ − 740
text {*
123
+ − 741
Unfortunately, also this function does \emph{not} work as expected, since
122
+ − 742
+ − 743
@{ML_response [display,gray] "is_nil @{term \"Nil\"}" "false"}
+ − 744
123
+ − 745
The problem is that on the ML-level the name of a constant is more
149
+ − 746
subtle than you might expect. The function @{ML is_all} worked correctly,
123
+ − 747
because @{term "All"} is such a fundamental constant, which can be referenced
+ − 748
by @{ML "Const (\"All\", some_type)" for some_type}. However, if you look at
122
+ − 749
+ − 750
@{ML_response [display,gray] "@{term \"Nil\"}" "Const (\"List.list.Nil\", \<dots>)"}
+ − 751
131
+ − 752
the name of the constant @{text "Nil"} depends on the theory in which the
128
+ − 753
term constructor is defined (@{text "List"}) and also in which datatype
+ − 754
(@{text "list"}). Even worse, some constants have a name involving
+ − 755
type-classes. Consider for example the constants for @{term "zero"} and
131
+ − 756
\mbox{@{text "(op *)"}}:
122
+ − 757
+ − 758
@{ML_response [display,gray] "(@{term \"0::nat\"}, @{term \"op *\"})"
126
+ − 759
"(Const (\"HOL.zero_class.zero\", \<dots>),
122
+ − 760
Const (\"HOL.times_class.times\", \<dots>))"}
+ − 761
123
+ − 762
While you could use the complete name, for example
+ − 763
@{ML "Const (\"List.list.Nil\", some_type)" for some_type}, for referring to or
122
+ − 764
matching against @{text "Nil"}, this would make the code rather brittle.
+ − 765
The reason is that the theory and the name of the datatype can easily change.
123
+ − 766
To make the code more robust, it is better to use the antiquotation
122
+ − 767
@{text "@{const_name \<dots>}"}. With this antiquotation you can harness the
123
+ − 768
variable parts of the constant's name. Therefore a functions for
+ − 769
matching against constants that have a polymorphic type should
+ − 770
be written as follows.
122
+ − 771
*}
+ − 772
+ − 773
ML{*fun is_nil_or_all (Const (@{const_name "Nil"}, _)) = true
+ − 774
| is_nil_or_all (Const (@{const_name "All"}, _) $ _) = true
+ − 775
| is_nil_or_all _ = false *}
+ − 776
+ − 777
text {*
131
+ − 778
Occasional you have to calculate what the ``base'' name of a given
124
+ − 779
constant is. For this you can use the function @{ML Sign.extern_const} or
163
2319cff107f0
removed rep_ss, and used dest_ss instead; some very slight changes to simple_inductive
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 780
@{ML Long_Name.base_name}. For example:
124
+ − 781
+ − 782
@{ML_response [display,gray] "Sign.extern_const @{theory} \"List.list.Nil\"" "\"Nil\""}
122
+ − 783
124
+ − 784
The difference between both functions is that @{ML extern_const in Sign} returns
163
2319cff107f0
removed rep_ss, and used dest_ss instead; some very slight changes to simple_inductive
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 785
the smallest name that is still unique, whereas @{ML base_name in Long_Name} always
124
+ − 786
strips off all qualifiers.
122
+ − 787
+ − 788
\begin{readmore}
162
+ − 789
Functions about naming are implemented in @{ML_file "Pure/General/name_space.ML"};
+ − 790
functions about signatures in @{ML_file "Pure/sign.ML"}.
122
+ − 791
\end{readmore}
186
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 792
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 793
Although types of terms can often be inferred, there are many
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 794
situations where you need to construct types manually, especially
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 795
when defining constants. For example the function returning a function
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 796
type is as follows:
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 797
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 798
*}
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 799
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 800
ML{*fun make_fun_type tau1 tau2 = Type ("fun", [tau1, tau2]) *}
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 801
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 802
text {* This can be equally written with the combinator @{ML "-->"} as: *}
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 803
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 804
ML{*fun make_fun_type tau1 tau2 = tau1 --> tau2 *}
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 805
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 806
text {*
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 807
A handy function for manipulating terms is @{ML map_types}: it takes a
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 808
function and applies it to every type in a term. You can, for example,
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 809
change every @{typ nat} in a term into an @{typ int} using the function:
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 810
*}
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 811
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 812
ML{*fun nat_to_int t =
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 813
(case t of
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 814
@{typ nat} => @{typ int}
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 815
| Type (s, ts) => Type (s, map nat_to_int ts)
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 816
| _ => t)*}
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 817
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 818
text {*
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 819
An example as follows:
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 820
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 821
@{ML_response_fake [display,gray]
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 822
"map_types nat_to_int @{term \"a = (1::nat)\"}"
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 823
"Const (\"op =\", \"int \<Rightarrow> int \<Rightarrow> bool\")
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 824
$ Free (\"a\", \"int\") $ Const (\"HOL.one_class.one\", \"int\")"}
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 825
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 826
(FIXME: readmore about types)
122
+ − 827
*}
162
+ − 828
122
+ − 829
124
+ − 830
section {* Type-Checking *}
+ − 831
+ − 832
text {*
+ − 833
131
+ − 834
You can freely construct and manipulate @{ML_type "term"}s and @{ML_type
+ − 835
typ}es, since they are just arbitrary unchecked trees. However, you
+ − 836
eventually want to see if a term is well-formed, or type-checks, relative to
+ − 837
a theory. Type-checking is done via the function @{ML cterm_of}, which
+ − 838
converts a @{ML_type term} into a @{ML_type cterm}, a \emph{certified}
+ − 839
term. Unlike @{ML_type term}s, which are just trees, @{ML_type "cterm"}s are
+ − 840
abstract objects that are guaranteed to be type-correct, and they can only
+ − 841
be constructed via ``official interfaces''.
+ − 842
124
+ − 843
+ − 844
Type-checking is always relative to a theory context. For now we use
+ − 845
the @{ML "@{theory}"} antiquotation to get hold of the current theory.
+ − 846
For example you can write:
+ − 847
149
+ − 848
@{ML_response_fake [display,gray] "cterm_of @{theory} @{term \"(a::nat) + b = c\"}" "a + b = c"}
124
+ − 849
+ − 850
This can also be written with an antiquotation:
+ − 851
+ − 852
@{ML_response_fake [display,gray] "@{cterm \"(a::nat) + b = c\"}" "a + b = c"}
+ − 853
+ − 854
Attempting to obtain the certified term for
+ − 855
+ − 856
@{ML_response_fake_both [display,gray] "@{cterm \"1 + True\"}" "Type unification failed \<dots>"}
+ − 857
+ − 858
yields an error (since the term is not typable). A slightly more elaborate
+ − 859
example that type-checks is:
+ − 860
+ − 861
@{ML_response_fake [display,gray]
+ − 862
"let
+ − 863
val natT = @{typ \"nat\"}
+ − 864
val zero = @{term \"0::nat\"}
+ − 865
in
+ − 866
cterm_of @{theory}
+ − 867
(Const (@{const_name plus}, natT --> natT --> natT) $ zero $ zero)
+ − 868
end" "0 + 0"}
+ − 869
186
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 870
In Isabelle not just terms need to be certified, but also types. For example,
178
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 871
you obtain the certified type for the Isablle type @{typ "nat \<Rightarrow> bool"} on
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 872
the ML-level as follows:
160
cc9359bfacf4
redefined the functions warning and tracing in order to properly match more antiquotations
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 873
cc9359bfacf4
redefined the functions warning and tracing in order to properly match more antiquotations
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 874
@{ML_response_fake [display,gray]
cc9359bfacf4
redefined the functions warning and tracing in order to properly match more antiquotations
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 875
"ctyp_of @{theory} (@{typ nat} --> @{typ bool})"
cc9359bfacf4
redefined the functions warning and tracing in order to properly match more antiquotations
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 876
"nat \<Rightarrow> bool"}
cc9359bfacf4
redefined the functions warning and tracing in order to properly match more antiquotations
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 877
cc9359bfacf4
redefined the functions warning and tracing in order to properly match more antiquotations
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 878
\begin{readmore}
cc9359bfacf4
redefined the functions warning and tracing in order to properly match more antiquotations
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 879
For functions related to @{ML_type cterm}s and @{ML_type ctyp}s see
cc9359bfacf4
redefined the functions warning and tracing in order to properly match more antiquotations
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 880
the file @{ML_file "Pure/thm.ML"}.
cc9359bfacf4
redefined the functions warning and tracing in order to properly match more antiquotations
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 881
\end{readmore}
cc9359bfacf4
redefined the functions warning and tracing in order to properly match more antiquotations
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 882
124
+ − 883
\begin{exercise}
+ − 884
Check that the function defined in Exercise~\ref{fun:revsum} returns a
+ − 885
result that type-checks.
+ − 886
\end{exercise}
+ − 887
178
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 888
Remember Isabelle foolows the Church-style typing for terms, i.e.~a term contains
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 889
enough typing information (constants, free variables and abstractions all have typing
124
+ − 890
information) so that it is always clear what the type of a term is.
+ − 891
Given a well-typed term, the function @{ML type_of} returns the
+ − 892
type of a term. Consider for example:
+ − 893
+ − 894
@{ML_response [display,gray]
+ − 895
"type_of (@{term \"f::nat \<Rightarrow> bool\"} $ @{term \"x::nat\"})" "bool"}
+ − 896
+ − 897
To calculate the type, this function traverses the whole term and will
128
+ − 898
detect any typing inconsistency. For examle changing the type of the variable
149
+ − 899
@{term "x"} from @{typ "nat"} to @{typ "int"} will result in the error message:
124
+ − 900
+ − 901
@{ML_response_fake [display,gray]
+ − 902
"type_of (@{term \"f::nat \<Rightarrow> bool\"} $ @{term \"x::int\"})"
+ − 903
"*** Exception- TYPE (\"type_of: type mismatch in application\" \<dots>"}
+ − 904
+ − 905
Since the complete traversal might sometimes be too costly and
149
+ − 906
not necessary, there is the function @{ML fastype_of}, which
+ − 907
also returns the type of a term.
124
+ − 908
+ − 909
@{ML_response [display,gray]
+ − 910
"fastype_of (@{term \"f::nat \<Rightarrow> bool\"} $ @{term \"x::nat\"})" "bool"}
+ − 911
177
+ − 912
However, efficiency is gained on the expense of skipping some tests. You
124
+ − 913
can see this in the following example
+ − 914
+ − 915
@{ML_response [display,gray]
+ − 916
"fastype_of (@{term \"f::nat \<Rightarrow> bool\"} $ @{term \"x::int\"})" "bool"}
+ − 917
149
+ − 918
where no error is detected.
124
+ − 919
+ − 920
Sometimes it is a bit inconvenient to construct a term with
+ − 921
complete typing annotations, especially in cases where the typing
+ − 922
information is redundant. A short-cut is to use the ``place-holder''
+ − 923
type @{ML "dummyT"} and then let type-inference figure out the
+ − 924
complete type. An example is as follows:
+ − 925
+ − 926
@{ML_response_fake [display,gray]
+ − 927
"let
126
+ − 928
val c = Const (@{const_name \"plus\"}, dummyT)
+ − 929
val o = @{term \"1::nat\"}
+ − 930
val v = Free (\"x\", dummyT)
124
+ − 931
in
126
+ − 932
Syntax.check_term @{context} (c $ o $ v)
124
+ − 933
end"
126
+ − 934
"Const (\"HOL.plus_class.plus\", \"nat \<Rightarrow> nat \<Rightarrow> nat\") $
+ − 935
Const (\"HOL.one_class.one\", \"nat\") $ Free (\"x\", \"nat\")"}
124
+ − 936
+ − 937
Instead of giving explicitly the type for the constant @{text "plus"} and the free
149
+ − 938
variable @{text "x"}, the type-inference filles in the missing information.
124
+ − 939
+ − 940
\begin{readmore}
+ − 941
See @{ML_file "Pure/Syntax/syntax.ML"} where more functions about reading,
160
cc9359bfacf4
redefined the functions warning and tracing in order to properly match more antiquotations
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 942
checking and pretty-printing of terms are defined. Fuctions related to the
cc9359bfacf4
redefined the functions warning and tracing in order to properly match more antiquotations
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 943
type inference are implemented in @{ML_file "Pure/type.ML"} and
cc9359bfacf4
redefined the functions warning and tracing in order to properly match more antiquotations
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 944
@{ML_file "Pure/type_infer.ML"}.
124
+ − 945
\end{readmore}
162
+ − 946
+ − 947
(FIXME: say something about sorts)
124
+ − 948
*}
+ − 949
+ − 950
2
+ − 951
section {* Theorems *}
+ − 952
+ − 953
text {*
50
+ − 954
Just like @{ML_type cterm}s, theorems are abstract objects of type @{ML_type thm}
122
+ − 955
that can only be build by going through interfaces. As a consequence, every proof
124
+ − 956
in Isabelle is correct by construction. This follows the tradition of the LCF approach
+ − 957
\cite{GordonMilnerWadsworth79}.
107
+ − 958
2
+ − 959
78
+ − 960
To see theorems in ``action'', let us give a proof on the ML-level for the following
+ − 961
statement:
10
+ − 962
*}
+ − 963
+ − 964
lemma
+ − 965
assumes assm\<^isub>1: "\<And>(x::nat). P x \<Longrightarrow> Q x"
+ − 966
and assm\<^isub>2: "P t"
13
+ − 967
shows "Q t" (*<*)oops(*>*)
10
+ − 968
+ − 969
text {*
185
+ − 970
The corresponding ML-code is as follows:
10
+ − 971
72
7b8c4fe235aa
added an antiquotation option [gray] for gray boxes around displays
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 972
@{ML_response_fake [display,gray]
42
+ − 973
"let
138
+ − 974
val assm1 = @{cprop \"\<And>(x::nat). P x \<Longrightarrow> Q x\"}
+ − 975
val assm2 = @{cprop \"(P::nat\<Rightarrow>bool) t\"}
10
+ − 976
+ − 977
val Pt_implies_Qt =
+ − 978
assume assm1
138
+ − 979
|> forall_elim @{cterm \"t::nat\"};
10
+ − 980
+ − 981
val Qt = implies_elim Pt_implies_Qt (assume assm2);
+ − 982
in
+ − 983
Qt
+ − 984
|> implies_intr assm2
+ − 985
|> implies_intr assm1
48
+ − 986
end" "\<lbrakk>\<And>x. P x \<Longrightarrow> Q x; P t\<rbrakk> \<Longrightarrow> Q t"}
12
+ − 987
21
+ − 988
This code-snippet constructs the following proof:
+ − 989
+ − 990
\[
+ − 991
\infer[(@{text "\<Longrightarrow>"}$-$intro)]{\vdash @{prop "(\<And>x. P x \<Longrightarrow> Q x) \<Longrightarrow> P t \<Longrightarrow> Q t"}}
+ − 992
{\infer[(@{text "\<Longrightarrow>"}$-$intro)]{@{prop "\<And>x. P x \<Longrightarrow> Q x"} \vdash @{prop "P t \<Longrightarrow> Q t"}}
+ − 993
{\infer[(@{text "\<Longrightarrow>"}$-$elim)]{@{prop "\<And>x. P x \<Longrightarrow> Q x"}, @{prop "P t"} \vdash @{prop "Q t"}}
+ − 994
{\infer[(@{text "\<And>"}$-$elim)]{@{prop "\<And>x. P x \<Longrightarrow> Q x"} \vdash @{prop "P t \<Longrightarrow> Q t"}}
+ − 995
{\infer[(assume)]{@{prop "\<And>x. P x \<Longrightarrow> Q x"} \vdash @{prop "\<And>x. P x \<Longrightarrow> Q x"}}{}}
+ − 996
&
+ − 997
\infer[(assume)]{@{prop "P t"} \vdash @{prop "P t"}}{}
+ − 998
}
+ − 999
}
+ − 1000
}
+ − 1001
\]
+ − 1002
102
5e309df58557
general cleaning up; deleted antiquotation ML_text; adjusted pathnames of various files in the distribution
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1003
However, while we obtained a theorem as result, this theorem is not
5e309df58557
general cleaning up; deleted antiquotation ML_text; adjusted pathnames of various files in the distribution
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1004
yet stored in Isabelle's theorem database. So it cannot be referenced later
128
+ − 1005
on. How to store theorems will be explained in Section~\ref{sec:storing}.
21
+ − 1006
13
+ − 1007
\begin{readmore}
50
+ − 1008
For the functions @{text "assume"}, @{text "forall_elim"} etc
13
+ − 1009
see \isccite{sec:thms}. The basic functions for theorems are defined in
+ − 1010
@{ML_file "Pure/thm.ML"}.
+ − 1011
\end{readmore}
12
+ − 1012
127
+ − 1013
(FIXME: how to add case-names to goal states - maybe in the next section)
10
+ − 1014
*}
+ − 1015
123
+ − 1016
section {* Theorem Attributes *}
+ − 1017
127
+ − 1018
text {*
133
+ − 1019
Theorem attributes are @{text "[simp]"}, @{text "[OF \<dots>]"}, @{text
136
+ − 1020
"[symmetric]"} and so on. Such attributes are \emph{neither} tags \emph{nor} flags
+ − 1021
annotated to theorems, but functions that do further processing once a
+ − 1022
theorem is proven. In particular, it is not possible to find out
+ − 1023
what are all theorems that have a given attribute in common, unless of course
133
+ − 1024
the function behind the attribute stores the theorems in a retrivable
151
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1025
datastructure.
127
+ − 1026
+ − 1027
If you want to print out all currently known attributes a theorem
+ − 1028
can have, you can use the function:
+ − 1029
+ − 1030
@{ML_response_fake [display,gray] "Attrib.print_attributes @{theory}"
+ − 1031
"COMP: direct composition with rules (no lifting)
+ − 1032
HOL.dest: declaration of Classical destruction rule
+ − 1033
HOL.elim: declaration of Classical elimination rule
+ − 1034
\<dots>"}
+ − 1035
136
+ − 1036
To explain how to write your own attribute, let us start with an extremely simple
+ − 1037
version of the attribute @{text "[symmetric]"}. The purpose of this attribute is
+ − 1038
to produce the ``symmetric'' version of an equation. The main function behind
+ − 1039
this attribute is
127
+ − 1040
*}
+ − 1041
133
+ − 1042
ML{*val my_symmetric = Thm.rule_attribute (fn _ => fn thm => thm RS @{thm sym})*}
+ − 1043
+ − 1044
text {*
136
+ − 1045
where the function @{ML "Thm.rule_attribute"} expects a function taking a
149
+ − 1046
context (which we ignore in the code above) and a theorem (@{text thm}), and
+ − 1047
returns another theorem (namely @{text thm} resolved with the lemma
+ − 1048
@{thm [source] sym}: @{thm sym[no_vars]}). The function @{ML "Thm.rule_attribute"} then returns
156
+ − 1049
an attribute.
136
+ − 1050
+ − 1051
Before we can use the attribute, we need to set it up. This can be done
178
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1052
using the function @{ML Attrib.setup} as follows.
133
+ − 1053
*}
+ − 1054
178
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1055
setup %gray {* Attrib.setup @{binding "my_sym"}
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1056
(Scan.succeed my_symmetric) "applying the sym rule"*}
133
+ − 1057
136
+ − 1058
text {*
149
+ − 1059
The attribute does not expect any further arguments (unlike @{text "[OF
+ − 1060
\<dots>]"}, for example, which can take a list of theorems as argument). Therefore
178
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1061
we use the parser @{ML Scan.succeed}. Later on we will also consider
149
+ − 1062
attributes taking further arguments. An example for the attribute @{text
+ − 1063
"[my_sym]"} is the proof
136
+ − 1064
*}
+ − 1065
+ − 1066
lemma test[my_sym]: "2 = Suc (Suc 0)" by simp
133
+ − 1067
+ − 1068
text {*
136
+ − 1069
which stores the theorem @{thm test} under the name @{thm [source] test}. We
+ − 1070
can also use the attribute when referring to this theorem.
+ − 1071
+ − 1072
\begin{isabelle}
+ − 1073
\isacommand{thm}~@{text "test[my_sym]"}\\
+ − 1074
@{text "> "}~@{thm test[my_sym]}
+ − 1075
\end{isabelle}
+ − 1076
151
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1077
The purpose of @{ML Thm.rule_attribute} is to directly manipulate theorems.
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1078
Another usage of attributes is to add and delete theorems from stored data.
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1079
For example the attribute @{text "[simp]"} adds or deletes a theorem from the
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1080
current simpset. For these applications, you can use @{ML Thm.declaration_attribute}.
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1081
To illustrate this function, let us introduce a reference containing a list
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1082
of theorems.
133
+ − 1083
*}
+ − 1084
151
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1085
ML{*val my_thms = ref ([]:thm list)*}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1086
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1087
text {*
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1088
A word of warning: such references must not be used in any code that
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1089
is meant to be more than just for testing purposes! Here it is only used
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1090
to illustrate matters. We will show later how to store data properly without
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1091
using references. The function @{ML Thm.declaration_attribute} expects us to
153
+ − 1092
provide two functions that add and delete theorems from this list.
+ − 1093
For this we use the two functions:
151
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1094
*}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1095
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1096
ML{*fun my_thms_add thm ctxt =
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1097
(my_thms := Thm.add_thm thm (!my_thms); ctxt)
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1098
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1099
fun my_thms_del thm ctxt =
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1100
(my_thms := Thm.del_thm thm (!my_thms); ctxt)*}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1101
133
+ − 1102
text {*
151
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1103
These functions take a theorem and a context and, for what we are explaining
156
+ − 1104
here it is sufficient that they just return the context unchanged. They change
151
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1105
however the reference @{ML my_thms}, whereby the function @{ML Thm.add_thm}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1106
adds a theorem if it is not already included in the list, and @{ML
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1107
Thm.del_thm} deletes one. Both functions use the predicate @{ML
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1108
Thm.eq_thm_prop} which compares theorems according to their proved
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1109
propositions (modulo alpha-equivalence).
133
+ − 1110
+ − 1111
156
+ − 1112
You can turn both functions into attributes using
151
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1113
*}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1114
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1115
ML{*val my_add = Thm.declaration_attribute my_thms_add
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1116
val my_del = Thm.declaration_attribute my_thms_del *}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1117
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1118
text {*
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1119
and set up the attributes as follows
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1120
*}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1121
178
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1122
setup %gray {* Attrib.setup @{binding "my_thms"}
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1123
(Attrib.add_del my_add my_del) "maintaining a list of my_thms" *}
151
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1124
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1125
text {*
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1126
Now if you prove the lemma attaching the attribute @{text "[my_thms]"}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1127
*}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1128
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1129
lemma trueI_2[my_thms]: "True" by simp
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1130
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1131
text {*
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1132
then you can see the lemma is added to the initially empty list.
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1133
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1134
@{ML_response_fake [display,gray]
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1135
"!my_thms" "[\"True\"]"}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1136
160
cc9359bfacf4
redefined the functions warning and tracing in order to properly match more antiquotations
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1137
You can also add theorems using the command \isacommand{declare}.
151
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1138
*}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1139
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1140
declare test[my_thms] trueI_2[my_thms add]
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1141
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1142
text {*
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1143
The @{text "add"} is the default operation and does not need
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1144
to be given. This declaration will cause the theorem list to be
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1145
updated as follows.
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1146
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1147
@{ML_response_fake [display,gray]
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1148
"!my_thms"
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1149
"[\"True\", \"Suc (Suc 0) = 2\"]"}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1150
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1151
The theorem @{thm [source] trueI_2} only appears once, since the
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1152
function @{ML Thm.add_thm} tests for duplicates, before extending
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1153
the list. Deletion from the list works as follows:
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1154
*}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1155
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1156
declare test[my_thms del]
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1157
156
+ − 1158
text {* After this, the theorem list is again:
151
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1159
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1160
@{ML_response_fake [display,gray]
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1161
"!my_thms"
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1162
"[\"True\"]"}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1163
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1164
We used in this example two functions declared as @{ML Thm.declaration_attribute},
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1165
but there can be any number of them. We just have to change the parser for reading
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1166
the arguments accordingly.
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1167
156
+ − 1168
However, as said at the beginning of this example, using references for storing theorems is
151
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1169
\emph{not} the received way of doing such things. The received way is to
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1170
start a ``data slot'' in a context by using the functor @{text GenericDataFun}:
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1171
*}
133
+ − 1172
151
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1173
ML {*structure Data = GenericDataFun
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1174
(type T = thm list
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1175
val empty = []
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1176
val extend = I
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1177
fun merge _ = Thm.merge_thms) *}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1178
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1179
text {*
156
+ − 1180
To use this data slot, you only have to change @{ML my_thms_add} and
151
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1181
@{ML my_thms_del} to:
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1182
*}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1183
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1184
ML{*val thm_add = Data.map o Thm.add_thm
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1185
val thm_del = Data.map o Thm.del_thm*}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1186
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1187
text {*
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1188
where @{ML Data.map} updates the data appropriately in the context. Since storing
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1189
theorems in a special list is such a common task, there is the functor @{text NamedThmsFun},
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1190
which does most of the work for you. To obtain such a named theorem lists, you just
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1191
declare
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1192
*}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1193
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1194
ML{*structure FooRules = NamedThmsFun
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1195
(val name = "foo"
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1196
val description = "Rules for foo"); *}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1197
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1198
text {*
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1199
and set up the @{ML_struct FooRules} with the command
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1200
*}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1201
177
+ − 1202
setup %gray {* FooRules.setup *}
151
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1203
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1204
text {*
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1205
This code declares a data slot where the theorems are stored,
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1206
an attribute @{text foo} (with the @{text add} and @{text del} options
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1207
for adding and deleting theorems) and an internal ML interface to retrieve and
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1208
modify the theorems.
133
+ − 1209
157
+ − 1210
Furthermore, the facts are made available on the user-level under the dynamic
156
+ − 1211
fact name @{text foo}. For example you can declare three lemmas to be of the kind
151
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1212
@{text foo} by:
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1213
*}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1214
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1215
lemma rule1[foo]: "A" sorry
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1216
lemma rule2[foo]: "B" sorry
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1217
lemma rule3[foo]: "C" sorry
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1218
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1219
text {* and undeclare the first one by: *}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1220
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1221
declare rule1[foo del]
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1222
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1223
text {* and query the remaining ones with:
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1224
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1225
\begin{isabelle}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1226
\isacommand{thm}~@{text "foo"}\\
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1227
@{text "> ?C"}\\
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1228
@{text "> ?B"}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1229
\end{isabelle}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1230
156
+ − 1231
On the ML-level the rules marked with @{text "foo"} can be retrieved
151
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1232
using the function @{ML FooRules.get}:
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1233
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1234
@{ML_response_fake [display,gray] "FooRules.get @{context}" "[\"?C\",\"?B\"]"}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1235
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1236
\begin{readmore}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1237
For more information see @{ML_file "Pure/Tools/named_thms.ML"} and also
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1238
the recipe in Section~\ref{recipe:storingdata} about storing arbitrary
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1239
data.
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1240
\end{readmore}
7e0bf13bf743
added more material to the attribute section; merged the recipe about named theorems into the main body; added a solution to an exercise in the conversion section
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1241
156
+ − 1242
(FIXME What are: @{text "theory_attributes"}, @{text "proof_attributes"}?)
133
+ − 1243
+ − 1244
+ − 1245
\begin{readmore}
+ − 1246
FIXME: @{ML_file "Pure/more_thm.ML"} @{ML_file "Pure/Isar/attrib.ML"}
+ − 1247
\end{readmore}
+ − 1248
*}
+ − 1249
127
+ − 1250
178
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1251
section {* Setups (TBD) *}
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1252
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1253
text {*
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1254
In the previous section we used \isacommand{setup} in order to make
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1255
a theorem attribute known to Isabelle. What happens behind the scenes
186
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1256
is that \isacommand{setup} expects a functions of type
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1257
@{ML_type "theory -> theory"}: the input theory is the current theory and the
178
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1258
output the theory where the theory attribute has been stored.
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1259
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1260
This is a fundamental principle in Isabelle. A similar situation occurs
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1261
for example with declaring constants. The function that declares a
186
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1262
constant on the ML-level is @{ML Sign.add_consts_i}.
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1263
If you write\footnote{Recall that ML-code needs to be
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1264
enclosed in \isacommand{ML}~@{text "\<verbopen> \<dots> \<verbclose>"}.}
178
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1265
*}
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1266
186
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1267
ML{*Sign.add_consts_i [(@{binding "BAR"}, @{typ "nat"}, NoSyn)] @{theory} *}
178
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1268
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1269
text {*
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1270
for declaring the constant @{text "BAR"} with type @{typ nat} and
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1271
run the code, then you indeed obtain a theory as result. But if you
186
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1272
query the constant on the Isabelle level using the command \isacommand{term}
178
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1273
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1274
\begin{isabelle}
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1275
\isacommand{term}~@{text [quotes] "BAR"}\\
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1276
@{text "> \"BAR\" :: \"'a\""}
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1277
\end{isabelle}
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1278
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1279
you do not obtain a constant of type @{typ nat}, but a free variable (printed in
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1280
blue) of polymorphic type. The problem is that the ML-expression above did
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1281
not register the declaration with the current theory. This is what the command
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1282
\isacommand{setup} is for. The constant is properly declared with
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1283
*}
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1284
186
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1285
setup %gray {* Sign.add_consts_i [(@{binding "BAR"}, @{typ "nat"}, NoSyn)] *}
178
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1286
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1287
text {*
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1288
Now
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1289
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1290
\begin{isabelle}
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1291
\isacommand{term}~@{text [quotes] "BAR"}\\
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1292
@{text "> \"BAR\" :: \"nat\""}
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1293
\end{isabelle}
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1294
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1295
returns a (black) constant with the type @{typ nat}.
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1296
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1297
A similar command is \isacommand{local\_setup}, which expects a function
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1298
of type @{ML_type "local_theory -> local_theory"}. Later on we will also
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1299
use the commands \isacommand{method\_setup} for installing methods in the
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1300
current theory and \isacommand{simproc\_setup} for adding new simprocs to
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1301
the current simpset.
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1302
*}
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1303
153
+ − 1304
section {* Theories, Contexts and Local Theories (TBD) *}
123
+ − 1305
126
+ − 1306
text {*
+ − 1307
There are theories, proof contexts and local theories (in this order, if you
+ − 1308
want to order them).
+ − 1309
+ − 1310
In contrast to an ordinary theory, which simply consists of a type
+ − 1311
signature, as well as tables for constants, axioms and theorems, a local
+ − 1312
theory also contains additional context information, such as locally fixed
+ − 1313
variables and local assumptions that may be used by the package. The type
+ − 1314
@{ML_type local_theory} is identical to the type of \emph{proof contexts}
+ − 1315
@{ML_type "Proof.context"}, although not every proof context constitutes a
+ − 1316
valid local theory.
178
fb8f22dd8ad0
adapted to latest Attrib.setup changes and more work on the simple induct chapter
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1317
*}
126
+ − 1318
153
+ − 1319
section {* Storing Theorems\label{sec:storing} (TBD) *}
123
+ − 1320
+ − 1321
text {* @{ML PureThy.add_thms_dynamic} *}
+ − 1322
100
+ − 1323
75
+ − 1324
126
+ − 1325
(* FIXME: some code below *)
89
+ − 1326
+ − 1327
(*<*)
163
2319cff107f0
removed rep_ss, and used dest_ss instead; some very slight changes to simple_inductive
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1328
(*
89
+ − 1329
setup {*
163
2319cff107f0
removed rep_ss, and used dest_ss instead; some very slight changes to simple_inductive
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1330
Sign.add_consts_i [(Binding"bar", @{typ "nat"},NoSyn)]
89
+ − 1331
*}
163
2319cff107f0
removed rep_ss, and used dest_ss instead; some very slight changes to simple_inductive
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1332
*)
89
+ − 1333
lemma "bar = (1::nat)"
+ − 1334
oops
+ − 1335
163
2319cff107f0
removed rep_ss, and used dest_ss instead; some very slight changes to simple_inductive
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1336
(*
89
+ − 1337
setup {*
+ − 1338
Sign.add_consts_i [("foo", @{typ "nat"},NoSyn)]
186
371e4375c994
made the Ackermann function example safer and included suggestions from MW
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1339
#> PureThy.add_defs false [((@{binding "foo_def"},
89
+ − 1340
Logic.mk_equals (Const ("FirstSteps.foo", @{typ "nat"}), @{term "1::nat"})), [])]
+ − 1341
#> snd
+ − 1342
*}
163
2319cff107f0
removed rep_ss, and used dest_ss instead; some very slight changes to simple_inductive
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1343
*)
2319cff107f0
removed rep_ss, and used dest_ss instead; some very slight changes to simple_inductive
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1344
(*
89
+ − 1345
lemma "foo = (1::nat)"
+ − 1346
apply(simp add: foo_def)
+ − 1347
done
+ − 1348
+ − 1349
thm foo_def
163
2319cff107f0
removed rep_ss, and used dest_ss instead; some very slight changes to simple_inductive
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1350
*)
89
+ − 1351
(*>*)
+ − 1352
153
+ − 1353
section {* Pretty-Printing (TBD) *}
+ − 1354
+ − 1355
text {*
163
2319cff107f0
removed rep_ss, and used dest_ss instead; some very slight changes to simple_inductive
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1356
@{ML Pretty.big_list},
2319cff107f0
removed rep_ss, and used dest_ss instead; some very slight changes to simple_inductive
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1357
@{ML Pretty.brk},
2319cff107f0
removed rep_ss, and used dest_ss instead; some very slight changes to simple_inductive
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1358
@{ML Pretty.block},
2319cff107f0
removed rep_ss, and used dest_ss instead; some very slight changes to simple_inductive
Christian Urban <urbanc@in.tum.de>
diff
changeset
+ − 1359
@{ML Pretty.chunks}
153
+ − 1360
*}
+ − 1361
+ − 1362
section {* Misc (TBD) *}
92
+ − 1363
+ − 1364
ML {*DatatypePackage.get_datatype @{theory} "List.list"*}
+ − 1365
196
+ − 1366
end