Results using cardinal arithmetic #
This file contains results using cardinal arithmetic that are not in the main cardinal theory files.
It has been separated out to not burden Matlib.Data.Set.Card
with extra imports.
Main results #
exists_union_disjoint_ncard_eq_of_even
: Given a sets
with an even cardinality, there exist disjoint setst
andu
such thatt ∪ u = s
andt.ncard = u.ncard
.exists_union_disjoint_cardinal_eq_iff
is the same, except using cardinal notation.
theorem
Set.Infinite.exists_union_disjoint_cardinal_eq_of_infinite
{α : Type u_1}
{s : Set α}
(h : s.Infinite)
:
∃ (t : Set α) (u : Set α), t ∪ u = s ∧ Disjoint t u ∧ Cardinal.mk ↑t = Cardinal.mk ↑u