| author | blanchet | 
| Wed, 01 Jun 2011 19:50:59 +0200 | |
| changeset 43139 | 9ed5d8ad8fa0 | 
| parent 41589 | bbd861837ebc | 
| child 46783 | 3e89a5cab8d7 | 
| permissions | -rw-r--r-- | 
| 14620 
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
 skalberg parents: 
14516diff
changeset | 1 | (* Title: HOL/Import/HOL4Syntax.thy | 
| 41589 | 2 | Author: Sebastian Skalberg, TU Muenchen | 
| 14620 
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
 skalberg parents: 
14516diff
changeset | 3 | *) | 
| 
1be590fd2422
Minor cleanup of headers and some speedup of the HOL4 import.
 skalberg parents: 
14516diff
changeset | 4 | |
| 41589 | 5 | theory HOL4Syntax | 
| 6 | imports HOL4Setup | |
| 7 | uses "import_syntax.ML" | |
| 8 | begin | |
| 14516 | 9 | |
| 10 | ML {* HOL4ImportSyntax.setup() *}
 | |
| 11 | ||
| 12 | end |