author | Christian Urban <urbanc@in.tum.de> |
Thu, 30 Oct 2008 13:36:51 +0100 | |
changeset 47 | 4daf913fdbe1 |
parent 46 | 81e2d73f7191 |
child 51 | c346c156a7cd |
permissions | -rw-r--r-- |
46
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
2 |
theory Antiquotes |
47
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
3 |
imports "../Base" |
46
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
4 |
begin |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
5 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
6 |
|
47
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
7 |
section {* Useful Document Antiquotations *} |
46
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
8 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
9 |
text {* |
47
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
10 |
{\bf Problem:} |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
11 |
How to keep ML-code included in a document in sync with the actual code.\smallskip |
46
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
12 |
|
47
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
13 |
{\bf Solution:} This can be achieved using document antiquotations.\smallskip |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
14 |
|
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
15 |
Document antiquotations are a convenient method for type-setting consitently |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
16 |
a group of items in a document. They can also be used for sophisticated |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
17 |
\LaTeX hacking. |
46
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
18 |
|
47
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
19 |
Below we give the code for two such |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
20 |
antiquotations that can be used to typeset ML-code and also to check whether |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
21 |
the code is actually compiles. In this way one can relatively easily |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
22 |
keep documents in sync with code. |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
23 |
|
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
24 |
We first describe the antiquotation @{text "@{ML_checked \"\<dots>\"}"} which |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
25 |
takes a piece of code as argument. This code is checked by sending |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
26 |
the ML-expression @{text "val _ = \<dots>"} containing the given code to the |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
27 |
ML-compiler (i.e.~the function @{ML "ML_Context.eval_in"}). The code |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
28 |
for this antiquotation is as follows: |
46
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
29 |
*} |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
30 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
31 |
ML {* |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
32 |
fun ml_val txt = "val _ = " ^ txt |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
33 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
34 |
fun output_ml ml src ctxt txt = |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
35 |
(ML_Context.eval_in (SOME ctxt) false Position.none (ml txt); |
47
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
36 |
ThyOutput.output_list (fn _ => fn s => Pretty.str s) src ctxt |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
37 |
(space_explode "\n" txt)) |
46
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
38 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
39 |
val _ = ThyOutput.add_commands |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
40 |
[("ML_checked", ThyOutput.args (Scan.lift Args.name) (output_ml ml_val))] |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
41 |
*} |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
42 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
43 |
text {* |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
44 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
45 |
Note that the parser @{ML "(Scan.lift Args.name)"} parses a string. If the |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
46 |
code is approved by the compiler, the output function |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
47 |
@{ML "ThyOutput.output_list (fn _ => fn s => Pretty.str s)"} |
47
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
48 |
pretty prints the code. This function expects that the code is a list of strings |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
49 |
according to the line breaks (therefore the |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
50 |
@{ML_open "(space_explode \"\\n\" txt)" for txt} which produces this list). |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
51 |
There are a number of options that are observed by @{ML ThyOutput.output_list} |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
52 |
when printing the code (for example @{text "[display]"} and @{text "[source]"}; |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
53 |
for more information about these options see \rsccite{sec:antiq}). |
46
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
54 |
|
47
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
55 |
Since we used the argument @{ML "Position.none"}, the compiler cannot give specific |
46
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
56 |
information about the line number where an error might have occurred. We |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
57 |
can improve this code slightly by writing |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
58 |
|
47
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
59 |
The second |
46
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
60 |
*} |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
61 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
62 |
ML {* |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
63 |
fun output_ml ml src ctxt (txt,pos) = |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
64 |
(ML_Context.eval_in (SOME ctxt) false pos (ml txt); |
47
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
65 |
ThyOutput.output_list (fn _ => fn s => Pretty.str s) src ctxt |
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
66 |
(space_explode "\n" txt)) |
46
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
67 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
68 |
val _ = ThyOutput.add_commands |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
69 |
[("ML_checked", ThyOutput.args |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
70 |
(Scan.lift (OuterParse.position Args.name)) (output_ml ml_val))] |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
71 |
*} |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
72 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
73 |
text {* |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
74 |
(FIXME: say something about OuterParse.position) |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
75 |
*} |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
76 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
77 |
ML {* |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
78 |
fun ml_pat (rhs, pat) = |
47
4daf913fdbe1
hakked latex so that it does not display ML {* *}; general tuning
Christian Urban <urbanc@in.tum.de>
parents:
46
diff
changeset
|
79 |
let val pat' = implode (map (fn "\<dots>" => "_" | s => s) (Symbol.explode pat)) |
46
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
80 |
in |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
81 |
"val " ^ pat' ^ " = " ^ rhs |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
82 |
end; |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
83 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
84 |
fun add_response_indicator txt = |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
85 |
map (fn s => "> " ^ s) (space_explode "\n" txt) |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
86 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
87 |
fun output_ml_response ml src ctxt ((lhs,pat),pos) = |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
88 |
(ML_Context.eval_in (SOME ctxt) false pos (ml (lhs,pat)); |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
89 |
let val txt = (space_explode "\n" lhs) @ (add_response_indicator pat) |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
90 |
in ThyOutput.output_list (fn _ => fn s => Pretty.str s) src ctxt txt end) |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
91 |
*} |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
92 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
93 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
94 |
(* |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
95 |
val _ = ThyOutput.add_commands |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
96 |
[("ML_response", |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
97 |
ThyOutput.args (Scan.lift (OuterParse.position (Args.name -- Args.name))) |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
98 |
(output_ml_response ml_pat)] |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
99 |
*) |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
100 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
101 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
102 |
ML {* |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
103 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
104 |
let |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
105 |
val i = 1 + 2 |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
106 |
in |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
107 |
i * i |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
108 |
end |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
109 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
110 |
*} |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
111 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
112 |
(* |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
113 |
A test: |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
114 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
115 |
@{ML_response [display] "true andalso false" "false"} |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
116 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
117 |
@{ML_response [display] |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
118 |
"let |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
119 |
val i = 1 + 2 |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
120 |
in |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
121 |
i * i |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
122 |
end" "9"} |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
123 |
*) |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
124 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
125 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
126 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
127 |
end |
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
128 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
129 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
130 |
|
81e2d73f7191
added a section about document antiquotations
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
131 |