Skip to content

Commit

Permalink
fix: Finpartition.atomise should not have [Fintype α] (#16617)
Browse files Browse the repository at this point in the history
Noticed by @b-mehta.
  • Loading branch information
Parcly-Taxel committed Sep 9, 2024
1 parent 5f1b34c commit 8c811c9
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions Mathlib/Order/Partition/Finpartition.lean
Original file line number Diff line number Diff line change
Expand Up @@ -548,6 +548,8 @@ lemma card_mod_card_parts_le : s.card % P.parts.card ≤ P.parts.card := by
rw [h, h']
· exact (Nat.mod_lt _ h).le

section Setoid

variable [Fintype α]

/-- A setoid over a finite type induces a finpartition of the type's elements,
Expand Down Expand Up @@ -587,6 +589,8 @@ theorem mem_part_ofSetoid_iff_rel {s : Setoid α} [DecidableRel s.r] {b : α} :
simp only [← hc, mem_univ, mem_filter, true_and] at this ⊢
exact ⟨s.trans (s.symm this), s.trans this⟩

end Setoid

section Atomise

/-- Cuts `s` along the finsets in `F`: Two elements of `s` will be in the same part if they are
Expand Down

0 comments on commit 8c811c9

Please sign in to comment.