src/HOL/Import/HOL4Syntax.thy
author huffman
Sun, 28 Aug 2011 20:56:49 -0700
changeset 44571 bd91b77c4cd6
parent 41589 bbd861837ebc
child 46783 3e89a5cab8d7
permissions -rw-r--r--
move class perfect_space into RealVector.thy; use not_open_singleton as perfect_space class axiom; generalize some lemmas to class perfect_space;

(*  Title:      HOL/Import/HOL4Syntax.thy
    Author:     Sebastian Skalberg, TU Muenchen
*)

theory HOL4Syntax
imports HOL4Setup
uses "import_syntax.ML"
begin

ML {* HOL4ImportSyntax.setup() *}

end