src/HOL/Record.thy
changeset 10309 a7f961fb62c6
parent 10093 44584c2b512b
child 10331 7411e4659d4a
--- a/src/HOL/Record.thy	Mon Oct 23 22:09:52 2000 +0200
+++ b/src/HOL/Record.thy	Mon Oct 23 22:10:36 2000 +0200
@@ -51,8 +51,7 @@
 (* type class for record extensions *)
 
 axclass more < "term"
-instance unit :: more
-  by intro_classes
+instance unit :: more ..
 
 
 (* initialize the package *)