Filters with countable intersection property #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we define countable_Inter_filter
to be the class of filters with the following
property: for any countable collection of sets s ∈ l
their intersection belongs to l
as well.
Two main examples are the residual
filter defined in topology.G_delta
and
the measure.ae
filter defined in measure_theory.measure_space
.
We reformulate the definition in terms of indexed intersection and in terms of filter.eventually
and provide instances for some basic constructions (⊥
, ⊤
, filter.principal
, filter.map
,
filter.comap
, has_inf.inf
). We also provide a custom constructor filter.of_countable_Inter
that deduces two axioms of a filter
from the countable intersection property.
Tags #
filter, countable
- countable_sInter_mem' : ∀ {S : set (set α)}, S.countable → (∀ (s : set α), s ∈ S → s ∈ l) → ⋂₀ S ∈ l
A filter l
has the countable intersection property if for any countable collection
of sets s ∈ l
their intersection belongs to l
as well.
Instances of this typeclass
- filter.countable_Inter_of_countable_Inter
- countable_Inter_filter_principal
- countable_Inter_filter_bot
- countable_Inter_filter_top
- filter.comap.countable_Inter_filter
- filter.map.countable_Inter_filter
- countable_Inter_filter_inf
- countable_Inter_filter_sup
- filter.countable_generate.countable_Inter_filter
- measure_theory.measure.ae.countable_Inter_filter
- residual.countable_Inter_filter
- countable_Inter_filter_residual
Construct a filter with countable intersection property. This constructor deduces
filter.univ_sets
and filter.inter_sets
from the countable intersection property.
Equations
- filter.of_countable_Inter l hp h_mono = {sets := l, univ_sets := _, sets_of_superset := h_mono, inter_sets := _}
Instances for filter.of_countable_Inter
Infimum of two countable_Inter_filter
s is a countable_Inter_filter
. This is useful, e.g.,
to automatically get an instance for residual α ⊓ 𝓟 s
.
Supremum of two countable_Inter_filter
s is a countable_Inter_filter
.
- basic : ∀ {α : Type u_2} {g : set (set α)} {s : set α}, s ∈ g → filter.countable_generate_sets g s
- univ : ∀ {α : Type u_2} {g : set (set α)}, filter.countable_generate_sets g set.univ
- superset : ∀ {α : Type u_2} {g : set (set α)} {s t : set α}, filter.countable_generate_sets g s → s ⊆ t → filter.countable_generate_sets g t
- Inter : ∀ {α : Type u_2} {g : set (set α)} {S : set (set α)}, S.countable → (∀ (s : set α), s ∈ S → filter.countable_generate_sets g s) → filter.countable_generate_sets g (⋂₀ S)
filter.countable_generate_sets g
is the (sets of the)
greatest countable_Inter_filter
containing g
.
filter.countable_generate g
is the greatest countable_Inter_filter
containing g
.
Equations
Instances for filter.countable_generate
A set is in the countable_Inter_filter
generated by g
if and only if
it contains a countable intersection of elements of g
.
countable_generate g
is the greatest countable_Inter_filter
containing g
.