Lemmas relating fintypes and order/lattice structure. #
theorem
Finset.sup_univ_eq_iSup
{α : Type u_2}
{β : Type u_3}
[Fintype α]
[CompleteLattice β]
(f : α → β)
:
A special case of Finset.sup_eq_iSup
that omits the useless x ∈ univ
binder.
theorem
Finset.inf_univ_eq_iInf
{α : Type u_2}
{β : Type u_3}
[Fintype α]
[CompleteLattice β]
(f : α → β)
:
A special case of Finset.inf_eq_iInf
that omits the useless x ∈ univ
binder.
theorem
Finite.exists_max
{α : Type u_2}
{β : Type u_3}
[Finite α]
[Nonempty α]
[LinearOrder β]
(f : α → β)
:
∃ (x₀ : α), ∀ (x : α), f x ≤ f x₀
theorem
Finite.exists_min
{α : Type u_2}
{β : Type u_3}
[Finite α]
[Nonempty α]
[LinearOrder β]
(f : α → β)
:
∃ (x₀ : α), ∀ (x : α), f x₀ ≤ f x