author | Christian Urban <urbanc@in.tum.de> |
Wed, 14 Oct 2009 02:32:53 +0200 | |
changeset 347 | 01e71cddf6a3 |
parent 346 | 0fea8b7a14a1 |
child 356 | 43df2d59fb98 |
permissions | -rw-r--r-- |
13
2b07da8b310d
polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1 |
|
2b07da8b310d
polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
2 |
theory Appendix |
346
0fea8b7a14a1
tuned the ML-output mechanism; tuned slightly the text
Christian Urban <urbanc@in.tum.de>
parents:
189
diff
changeset
|
3 |
imports Base |
13
2b07da8b310d
polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
4 |
begin |
2b07da8b310d
polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
5 |
|
346
0fea8b7a14a1
tuned the ML-output mechanism; tuned slightly the text
Christian Urban <urbanc@in.tum.de>
parents:
189
diff
changeset
|
6 |
(*<*) |
0fea8b7a14a1
tuned the ML-output mechanism; tuned slightly the text
Christian Urban <urbanc@in.tum.de>
parents:
189
diff
changeset
|
7 |
setup{* |
0fea8b7a14a1
tuned the ML-output mechanism; tuned slightly the text
Christian Urban <urbanc@in.tum.de>
parents:
189
diff
changeset
|
8 |
open_file_with_prelude |
0fea8b7a14a1
tuned the ML-output mechanism; tuned slightly the text
Christian Urban <urbanc@in.tum.de>
parents:
189
diff
changeset
|
9 |
"Recipes_Code.thy" |
0fea8b7a14a1
tuned the ML-output mechanism; tuned slightly the text
Christian Urban <urbanc@in.tum.de>
parents:
189
diff
changeset
|
10 |
["theory Recipes", "imports Main", "begin"] |
0fea8b7a14a1
tuned the ML-output mechanism; tuned slightly the text
Christian Urban <urbanc@in.tum.de>
parents:
189
diff
changeset
|
11 |
*} |
0fea8b7a14a1
tuned the ML-output mechanism; tuned slightly the text
Christian Urban <urbanc@in.tum.de>
parents:
189
diff
changeset
|
12 |
(*>*) |
182
4d0e2edd476d
added hyperlinks for every file pointer
Christian Urban <urbanc@in.tum.de>
parents:
168
diff
changeset
|
13 |
|
13
2b07da8b310d
polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
14 |
text {* \appendix *} |
2b07da8b310d
polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
15 |
|
129
e0d368a45537
started a section about simprocs
Christian Urban <urbanc@in.tum.de>
parents:
73
diff
changeset
|
16 |
|
13
2b07da8b310d
polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
17 |
chapter {* Recipes *} |
2b07da8b310d
polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
18 |
|
131 | 19 |
text {* |
184 | 20 |
Possible topics: |
162
3fb9f820a294
some additions to the simplifier section and general tuning
Christian Urban <urbanc@in.tum.de>
parents:
131
diff
changeset
|
21 |
|
168
009ca4807baa
polished somewhat the recipes and solutions
Christian Urban <urbanc@in.tum.de>
parents:
164
diff
changeset
|
22 |
\begin{itemize} |
009ca4807baa
polished somewhat the recipes and solutions
Christian Urban <urbanc@in.tum.de>
parents:
164
diff
changeset
|
23 |
\item translations/print translations; |
162
3fb9f820a294
some additions to the simplifier section and general tuning
Christian Urban <urbanc@in.tum.de>
parents:
131
diff
changeset
|
24 |
@{ML "ProofContext.print_syntax"} |
131 | 25 |
|
168
009ca4807baa
polished somewhat the recipes and solutions
Christian Urban <urbanc@in.tum.de>
parents:
164
diff
changeset
|
26 |
\item user space type systems (in the form that already exists) |
164
3f617d7a2691
more work on simple_inductive
Christian Urban <urbanc@in.tum.de>
parents:
162
diff
changeset
|
27 |
|
184 | 28 |
\item unification and typing algorithms |
29 |
(@{ML_file "Pure/pattern.ML"} implements HOPU) |
|
164
3f617d7a2691
more work on simple_inductive
Christian Urban <urbanc@in.tum.de>
parents:
162
diff
changeset
|
30 |
|
168
009ca4807baa
polished somewhat the recipes and solutions
Christian Urban <urbanc@in.tum.de>
parents:
164
diff
changeset
|
31 |
\item useful datastructures: discrimination nets, association lists |
009ca4807baa
polished somewhat the recipes and solutions
Christian Urban <urbanc@in.tum.de>
parents:
164
diff
changeset
|
32 |
\end{itemize} |
131 | 33 |
*} |
34 |
||
168
009ca4807baa
polished somewhat the recipes and solutions
Christian Urban <urbanc@in.tum.de>
parents:
164
diff
changeset
|
35 |
end |