src/HOL/Library/Quotient.thy
changeset 12338 de0f4a63baa5
parent 11549 e7265e70fd7c
child 12371 80ca9058db95
--- a/src/HOL/Library/Quotient.thy	Sat Dec 01 18:51:46 2001 +0100
+++ b/src/HOL/Library/Quotient.thy	Sat Dec 01 18:52:32 2001 +0100
@@ -23,7 +23,7 @@
  "\<sim> :: 'a => 'a => bool"}.
 *}
 
-axclass eqv \<subseteq> "term"
+axclass eqv \<subseteq> type
 consts
   eqv :: "('a::eqv) => 'a => bool"    (infixl "\<sim>" 50)