Filter.atTop
and Filter.atBot
filters and finite sets. #
theorem
Monotone.tendsto_atTop_finset
{α : Type u_3}
{β : Type u_4}
[Preorder β]
{f : β → Finset α}
(h : Monotone f)
(h' : ∀ (x : α), ∃ (n : β), x ∈ f n)
:
Alias of Filter.tendsto_atTop_finset_of_monotone
.
If f
is a monotone sequence of Finset
s and each x
belongs to one of f n
, then
Tendsto f atTop atTop
.
theorem
Filter.tendsto_finset_image_atTop_atTop
{β : Type u_4}
{γ : Type u_5}
[DecidableEq β]
{i : β → γ}
{j : γ → β}
(h : Function.LeftInverse j i)
:
theorem
Filter.tendsto_finset_preimage_atTop_atTop
{α : Type u_3}
{β : Type u_4}
{f : α → β}
(hf : Function.Injective f)
: