src/HOL/Import/HOL4Syntax.thy
author skalberg
Sun, 04 Apr 2004 15:34:14 +0200
changeset 14518 c3019a66180f
parent 14516 a183dec876ab
child 14620 1be590fd2422
permissions -rw-r--r--
Added a number of explicit type casts and delayed evaluations (all seemingly needless) so that SML/NJ 110.9.1 would accept the importer...

theory HOL4Syntax = HOL4Setup
  files "import_syntax.ML":

ML {* HOL4ImportSyntax.setup() *}

end