improved handling of polymorphic quotient types, by avoiding comparing types that will generally differ in the polymorphic case
(* Title: HOL/Import/HOL4Syntax.thy
Author: Sebastian Skalberg, TU Muenchen
*)
theory HOL4Syntax
imports HOL4Setup
uses "import_syntax.ML"
begin
ML {* HOL4ImportSyntax.setup() *}
end