Skip to content

Commit

Permalink
feat(data/setoid/partition): sUnion _classes (#2936)
Browse files Browse the repository at this point in the history
  • Loading branch information
ChrisHughes24 committed Jun 3, 2020
1 parent c3221f7 commit ed91bb2
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions src/data/setoid/partition.lean
Expand Up @@ -113,6 +113,9 @@ theorem mk_classes_classes (r : setoid α) :
ext' $ λ x y, ⟨λ h, r.symm' (h {z | r.rel z x} (r.mem_classes x) $ r.refl' x),
λ h b hb hx, eq_of_mem_classes (r.mem_classes x) (r.refl' x) hb hx ▸ r.symm' h⟩

@[simp] theorem sUnion_classes (r : setoid α) : ⋃₀ r.classes = set.univ :=
set.eq_univ_of_forall $ λ x, set.mem_sUnion.2 ⟨{ y | r.rel y x }, ⟨x, rfl⟩, setoid.refl _⟩

section partition

/-- A collection `c : set (set α)` of sets is a partition of `α` into pairwise
Expand Down

0 comments on commit ed91bb2

Please sign in to comment.