(Co)product of a family of filters #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we define two filters on Π i, α i
and prove some basic properties of these filters.
-
filter.pi (f : Π i, filter (α i))
to be the maximal filter onΠ i, α i
such that∀ i, filter.tendsto (function.eval i) (filter.pi f) (f i)
. It is defined asΠ i, filter.comap (function.eval i) (f i)
. This is a generalization offilter.prod
to indexed products. -
filter.Coprod (f : Π i, filter (α i))
: a generalization offilter.coprod
; it is the supremum ofcomap (eval i) (f i)
.
@[protected, instance]
def
filter.pi.is_countably_generated
{ι : Type u_1}
{α : ι → Type u_2}
{f : Π (i : ι), filter (α i)}
[countable ι]
[∀ (i : ι), (f i).is_countably_generated] :
theorem
filter.tendsto_eval_pi
{ι : Type u_1}
{α : ι → Type u_2}
(f : Π (i : ι), filter (α i))
(i : ι) :
filter.tendsto (function.eval i) (filter.pi f) (f i)
theorem
filter.le_pi
{ι : Type u_1}
{α : ι → Type u_2}
{f : Π (i : ι), filter (α i)}
{g : filter (Π (i : ι), α i)} :
g ≤ filter.pi f ↔ ∀ (i : ι), filter.tendsto (function.eval i) g (f i)
@[simp]
theorem
filter.map_eval_pi
{ι : Type u_1}
{α : ι → Type u_2}
(f : Π (i : ι), filter (α i))
[∀ (i : ι), (f i).ne_bot]
(i : ι) :
filter.map (function.eval i) (filter.pi f) = f i
n
-ary coproducts of filters #
@[protected]
Coproduct of filters.
Equations
- filter.Coprod f = ⨆ (i : ι), filter.comap (function.eval i) (f i)
Instances for filter.Coprod
@[simp]
theorem
filter.Coprod_mono
{ι : Type u_1}
{α : ι → Type u_2}
{f₁ f₂ : Π (i : ι), filter (α i)}
(hf : ∀ (i : ι), f₁ i ≤ f₂ i) :
filter.Coprod f₁ ≤ filter.Coprod f₂
theorem
filter.map_pi_map_Coprod_le
{ι : Type u_1}
{α : ι → Type u_2}
{f : Π (i : ι), filter (α i)}
{β : ι → Type u_3}
{m : Π (i : ι), α i → β i} :
filter.map (λ (k : Π (i : ι), α i) (i : ι), m i (k i)) (filter.Coprod f) ≤ filter.Coprod (λ (i : ι), filter.map (m i) (f i))
theorem
filter.tendsto.pi_map_Coprod
{ι : Type u_1}
{α : ι → Type u_2}
{f : Π (i : ι), filter (α i)}
{β : ι → Type u_3}
{m : Π (i : ι), α i → β i}
{g : Π (i : ι), filter (β i)}
(h : ∀ (i : ι), filter.tendsto (m i) (f i) (g i)) :
filter.tendsto (λ (k : Π (i : ι), α i) (i : ι), m i (k i)) (filter.Coprod f) (filter.Coprod g)