author | haftmann |
Wed, 07 Oct 2009 14:01:26 +0200 | |
changeset 32887 | 85e7ab9020ba |
parent 16417 | 9bc16273c2d4 |
child 41589 | bbd861837ebc |
permissions | -rw-r--r-- |
14620
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
skalberg
parents:
14516
diff
changeset
|
1 |
(* Title: HOL/Import/HOL4Syntax.thy |
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
skalberg
parents:
14516
diff
changeset
|
2 |
ID: $Id$ |
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
skalberg
parents:
14516
diff
changeset
|
3 |
Author: Sebastian Skalberg (TU Muenchen) |
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
skalberg
parents:
14516
diff
changeset
|
4 |
*) |
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
skalberg
parents:
14516
diff
changeset
|
5 |
|
16417 | 6 |
theory HOL4Syntax imports HOL4Setup |
7 |
uses "import_syntax.ML" begin |
|
14516 | 8 |
|
9 |
ML {* HOL4ImportSyntax.setup() *} |
|
10 |
||
11 |
end |