| author | ballarin | 
| Thu, 24 Mar 2005 16:34:15 +0100 | |
| changeset 15622 | 4723248c982b | 
| parent 14620 | 1be590fd2422 | 
| child 16417 | 9bc16273c2d4 | 
| 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  | 
|
| 14516 | 6  | 
theory HOL4Syntax = HOL4Setup  | 
7  | 
files "import_syntax.ML":  | 
|
8  | 
||
9  | 
ML {* HOL4ImportSyntax.setup() *}
 | 
|
10  | 
||
11  | 
end  |