author | wenzelm |
Wed, 06 Sep 2000 16:54:12 +0200 | |
changeset 9876 | a069795f1060 |
parent 9854 | a1383b55ac05 |
child 10261 | bb2f1e859177 |
permissions | -rw-r--r-- |
9619 | 1 |
|
2 |
(*theory Main includes everything; note that theory |
|
3 |
PreList already includes most HOL theories*) |
|
4 |
||
9650
6f0b89f2a1f9
Main now new-style theory; added Main.ML for compatibility;
wenzelm
parents:
9619
diff
changeset
|
5 |
theory Main = Map + String: |
6f0b89f2a1f9
Main now new-style theory; added Main.ML for compatibility;
wenzelm
parents:
9619
diff
changeset
|
6 |
|
9854 | 7 |
(*actually belongs to theory List*) |
9768 | 8 |
lemmas [mono] = lists_mono |
9876 | 9 |
lemmas [recdef_cong] = map_cong |
9768 | 10 |
|
9650
6f0b89f2a1f9
Main now new-style theory; added Main.ML for compatibility;
wenzelm
parents:
9619
diff
changeset
|
11 |
end |