author | Christian Urban <urbanc@in.tum.de> |
Tue, 10 Mar 2009 13:20:46 +0000 | |
changeset 164 | 3f617d7a2691 |
parent 162 | 3fb9f820a294 |
child 168 | 009ca4807baa |
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 |
2b07da8b310d
polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
3 |
imports Main |
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 |
|
2b07da8b310d
polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
6 |
text {* \appendix *} |
2b07da8b310d
polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
7 |
|
129
e0d368a45537
started a section about simprocs
Christian Urban <urbanc@in.tum.de>
parents:
73
diff
changeset
|
8 |
|
13
2b07da8b310d
polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
9 |
chapter {* Recipes *} |
2b07da8b310d
polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
10 |
|
131 | 11 |
text {* |
162
3fb9f820a294
some additions to the simplifier section and general tuning
Christian Urban <urbanc@in.tum.de>
parents:
131
diff
changeset
|
12 |
Possible further topics: |
3fb9f820a294
some additions to the simplifier section and general tuning
Christian Urban <urbanc@in.tum.de>
parents:
131
diff
changeset
|
13 |
|
3fb9f820a294
some additions to the simplifier section and general tuning
Christian Urban <urbanc@in.tum.de>
parents:
131
diff
changeset
|
14 |
translations/print translations |
3fb9f820a294
some additions to the simplifier section and general tuning
Christian Urban <urbanc@in.tum.de>
parents:
131
diff
changeset
|
15 |
|
3fb9f820a294
some additions to the simplifier section and general tuning
Christian Urban <urbanc@in.tum.de>
parents:
131
diff
changeset
|
16 |
@{ML "ProofContext.print_syntax"} |
131 | 17 |
|
162
3fb9f820a294
some additions to the simplifier section and general tuning
Christian Urban <urbanc@in.tum.de>
parents:
131
diff
changeset
|
18 |
user space type systems (in the form that already exists) |
3fb9f820a294
some additions to the simplifier section and general tuning
Christian Urban <urbanc@in.tum.de>
parents:
131
diff
changeset
|
19 |
|
3fb9f820a294
some additions to the simplifier section and general tuning
Christian Urban <urbanc@in.tum.de>
parents:
131
diff
changeset
|
20 |
unification and typing algorithms |
164
3f617d7a2691
more work on simple_inductive
Christian Urban <urbanc@in.tum.de>
parents:
162
diff
changeset
|
21 |
|
3f617d7a2691
more work on simple_inductive
Christian Urban <urbanc@in.tum.de>
parents:
162
diff
changeset
|
22 |
useful datastructures: |
3f617d7a2691
more work on simple_inductive
Christian Urban <urbanc@in.tum.de>
parents:
162
diff
changeset
|
23 |
|
3f617d7a2691
more work on simple_inductive
Christian Urban <urbanc@in.tum.de>
parents:
162
diff
changeset
|
24 |
discrimination nets |
3f617d7a2691
more work on simple_inductive
Christian Urban <urbanc@in.tum.de>
parents:
162
diff
changeset
|
25 |
|
3f617d7a2691
more work on simple_inductive
Christian Urban <urbanc@in.tum.de>
parents:
162
diff
changeset
|
26 |
association lists |
131 | 27 |
*} |
28 |
||
13
2b07da8b310d
polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
29 |
end |
2b07da8b310d
polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
30 |
|
2b07da8b310d
polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
31 |
|
2b07da8b310d
polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
32 |
|
2b07da8b310d
polished and added a subdirectory for the recipes
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
33 |