| author | wenzelm |
| Sun, 07 Feb 2016 19:43:40 +0100 | |
| changeset 62271 | 4cfe65cfd369 |
| parent 62270 | 77e3ffb5aeb3 |
| child 62312 | 5e5a881ebc12 |
| permissions | -rw-r--r-- |
| 61656 | 1 |
(*:maxLineLen=78:*) |
2 |
||
| 42651 | 3 |
theory Base |
4 |
imports Pure |
|
| 62270 | 5 |
keywords "\<proof>" :: "qed" % "proof" |
| 42651 | 6 |
begin |
7 |
||
| 62270 | 8 |
ML \<open> |
9 |
Outer_Syntax.command @{command_keyword "\<proof>"} "dummy proof"
|
|
10 |
(Scan.succeed Isar_Cmd.skip_proof); |
|
11 |
\<close> |
|
12 |
||
|
48958
12afbf6eb7f9
more standard document preparation within session context;
wenzelm
parents:
48956
diff
changeset
|
13 |
ML_file "../antiquote_setup.ML" |
| 42651 | 14 |
|
15 |
end |