src/HOL/Integ/Equiv.thy
changeset 12398 9c27f28c8f5a
parent 10834 a7897aebbffc
child 13482 2bb7200a99cf
--- a/src/HOL/Integ/Equiv.thy	Thu Dec 06 00:39:40 2001 +0100
+++ b/src/HOL/Integ/Equiv.thy	Thu Dec 06 00:40:04 2001 +0100
@@ -6,7 +6,7 @@
 Equivalence relations in Higher-Order Set Theory 
 *)
 
-Equiv = Relation + Finite + 
+Equiv = Relation + Finite_Set +
 constdefs
   equiv    :: "['a set, ('a*'a) set] => bool"
     "equiv A r == refl A r & sym(r) & trans(r)"