Equations
- instFintypeSum α β = { elems := Finset.univ.disjSum Finset.univ, complete := ⋯ }
theorem
image_subtype_ne_univ_eq_image_erase
{α : Type u_1}
{β : Type u_2}
[Fintype α]
[DecidableEq β]
(k : β)
(b : α → β)
:
Finset.image (fun (i : { a : α // b a ≠ k }) => b ↑i) Finset.univ = (Finset.image b Finset.univ).erase k
theorem
image_subtype_univ_ssubset_image_univ
{α : Type u_1}
{β : Type u_2}
[Fintype α]
[DecidableEq β]
(k : β)
(b : α → β)
(hk : k ∈ Finset.image b Finset.univ)
(p : β → Prop)
[DecidablePred p]
(hp : ¬p k)
:
Finset.image (fun (i : { a : α // p (b a) }) => b ↑i) Finset.univ ⊂ Finset.image b Finset.univ
theorem
Finset.exists_equiv_extend_of_card_eq
{α : Type u_1}
{β : Type u_2}
[Fintype α]
[DecidableEq β]
{t : Finset β}
(hαt : Fintype.card α = t.card)
{s : Finset α}
{f : α → β}
(hfst : image f s ⊆ t)
(hfs : Set.InjOn f ↑s)
:
Any injection from a finset s
in a fintype α
to a finset t
of the same cardinality as α
can be extended to a bijection between α
and t
.
theorem
Set.MapsTo.exists_equiv_extend_of_card_eq
{α : Type u_1}
{β : Type u_2}
[Fintype α]
{t : Finset β}
(hαt : Fintype.card α = t.card)
{s : Set α}
{f : α → β}
(hfst : MapsTo f s ↑t)
(hfs : InjOn f s)
:
Any injection from a set s
in a fintype α
to a finset t
of the same cardinality as α
can be extended to a bijection between α
and t
.