changeset 15131 | c69542757a4d |
parent 15108 | 492e5f3a8571 |
child 15140 | 322485b816ac |
--- a/src/HOL/Integ/Equiv.thy Mon Aug 16 14:21:54 2004 +0200 +++ b/src/HOL/Integ/Equiv.thy Mon Aug 16 14:22:27 2004 +0200 @@ -6,7 +6,9 @@ header {* Equivalence relations in Higher-Order Set Theory *} -theory Equiv = Relation + Finite_Set: +theory Equiv +import Relation Finite_Set +begin subsection {* Equivalence relations *}