Put in minimal simpset to avoid excessive simplification,
just as in revision 1.9 of HOL/indrule.ML
(* Title: HOL/AxClasses/Tutorial/Sigs.thy
ID: $Id$
Author: Markus Wenzel, TU Muenchen
Some polymorphic constants for the 'signature' parts of axclasses.
*)
Sigs = HOL +
consts
"<*>" :: "['a, 'a] => 'a" (infixl 70)
"inv" :: "'a => 'a"
"1" :: "'a" ("1")
end