Skip to content

Commit

Permalink
DecidableEq no longer needed
Browse files Browse the repository at this point in the history
  • Loading branch information
madvorak committed Jan 3, 2025
1 parent 1be3068 commit 61b2a51
Showing 1 changed file with 1 addition and 2 deletions.
3 changes: 1 addition & 2 deletions Mathlib/Data/Finset/Card.lean
Original file line number Diff line number Diff line change
Expand Up @@ -579,8 +579,7 @@ lemma exists_subsuperset_card_eq (hst : s ⊆ t) (hsn : #s ≤ n) (hnt : n ≤ #
lemma exists_subset_card_eq (hns : n ≤ #s) : ∃ t ⊆ s, #t = n := by
simpa using exists_subsuperset_card_eq s.empty_subset (by simp) hns

lemma of_cardinality_between_of_disjoint [DecidableEq α] (hs : #s < n) (hn : n ≤ #s + #t)
(hst : Disjoint s t) :
lemma of_cardinality_between_of_disjoint (hs : #s < n) (hn : n ≤ #s + #t) (hst : Disjoint s t) :
∃ (x : Finset α) (hxs : Disjoint x s), #(x.disjUnion s hxs) = n ∧ Nonempty x := by
have hnst : n - #s ≤ #t := by omega
obtain ⟨x, hxt, hxn⟩ := Finset.exists_subset_card_eq hnst
Expand Down

0 comments on commit 61b2a51

Please sign in to comment.