13
|
1 |
|
|
2 |
theory Appendix
|
346
|
3 |
imports Base
|
13
|
4 |
begin
|
|
5 |
|
346
|
6 |
(*<*)
|
|
7 |
setup{*
|
|
8 |
open_file_with_prelude
|
|
9 |
"Recipes_Code.thy"
|
|
10 |
["theory Recipes", "imports Main", "begin"]
|
|
11 |
*}
|
|
12 |
(*>*)
|
182
|
13 |
|
13
|
14 |
text {* \appendix *}
|
|
15 |
|
129
|
16 |
|
13
|
17 |
chapter {* Recipes *}
|
|
18 |
|
131
|
19 |
text {*
|
184
|
20 |
Possible topics:
|
162
|
21 |
|
168
|
22 |
\begin{itemize}
|
|
23 |
\item translations/print translations;
|
475
|
24 |
@{ML "Proof_Context.print_syntax"}
|
131
|
25 |
|
168
|
26 |
\item user space type systems (in the form that already exists)
|
164
|
27 |
|
407
|
28 |
\item useful datastructures: discrimination nets, graphs, association lists
|
356
|
29 |
|
|
30 |
\item Brief history of Isabelle
|
168
|
31 |
\end{itemize}
|
131
|
32 |
*}
|
|
33 |
|
168
|
34 |
end |