src/HOL/Equiv_Relations.thy
changeset 66364 fa3247e6ee4b
parent 63653 4453cfb745e5
child 67399 eab6ce8368fa
equal deleted inserted replaced
66363:8aca34dbe195 66364:fa3247e6ee4b
     3 *)
     3 *)
     4 
     4 
     5 section \<open>Equivalence Relations in Higher-Order Set Theory\<close>
     5 section \<open>Equivalence Relations in Higher-Order Set Theory\<close>
     6 
     6 
     7 theory Equiv_Relations
     7 theory Equiv_Relations
     8   imports Groups_Big Relation
     8   imports Groups_Big
     9 begin
     9 begin
    10 
    10 
    11 subsection \<open>Equivalence relations -- set version\<close>
    11 subsection \<open>Equivalence relations -- set version\<close>
    12 
    12 
    13 definition equiv :: "'a set \<Rightarrow> ('a \<times> 'a) set \<Rightarrow> bool"
    13 definition equiv :: "'a set \<Rightarrow> ('a \<times> 'a) set \<Rightarrow> bool"