Relating Finset.biUnion
with lattice operations #
This file shows Finset.biUnion
could alternatively be defined in terms of Finset.sup
.
TODO #
Remove Finset.biUnion
in favour of Finset.sup
.
@[simp]
theorem
Finset.sup_biUnion
{α : Type u_2}
{β : Type u_3}
{γ : Type u_4}
{f : β → α}
[SemilatticeSup α]
[OrderBot α]
[DecidableEq β]
(s : Finset γ)
(t : γ → Finset β)
:
@[simp]
theorem
Finset.inf_biUnion
{α : Type u_2}
{β : Type u_3}
{γ : Type u_4}
{f : β → α}
[SemilatticeInf α]
[OrderTop α]
[DecidableEq β]
(s : Finset γ)
(t : γ → Finset β)
:
theorem
Finset.sup_eq_biUnion
{α : Type u_7}
{β : Type u_8}
[DecidableEq β]
(s : Finset α)
(t : α → Finset β)
: