Baire theorem #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In a complete metric space, a countable intersection of dense open subsets is dense.
The good concept underlying the theorem is that of a Gδ set, i.e., a countable intersection of open sets. Then Baire theorem can also be formulated as the fact that a countable intersection of dense Gδ sets is a dense Gδ set. We prove Baire theorem, giving several different formulations that can be handy. We also prove the important consequence that, if the space is covered by a countable union of closed sets, then the union of their interiors is dense.
We also prove that in Baire spaces, the residual sets are exactly those containing a dense Gδ set.
- baire_property : ∀ (f : ℕ → set α), (∀ (n : ℕ), is_open (f n)) → (∀ (n : ℕ), dense (f n)) → dense (⋂ (n : ℕ), f n)
The property baire_space α means that the topological space α has the Baire property:
any countable intersection of open dense subsets is dense.
Formulated here when the source space is ℕ (and subsumed below by dense_Inter_of_open working
with any encodable source space).
Instances of this typeclass
Baire theorems asserts that various topological spaces have the Baire property. Two versions of these theorems are given. The first states that complete pseudo_emetric spaces are Baire.
The second theorem states that locally compact spaces are Baire.
Baire theorem: a countable intersection of dense open sets is dense. Formulated here with an index set which is a countable set in any type.
Baire theorem: a countable intersection of dense open sets is dense. Formulated here with an index set which is an encodable type.
Baire theorem: a countable intersection of dense Gδ sets is dense. Formulated here with an index set which is an encodable type.
Baire theorem: a countable intersection of dense Gδ sets is dense. Formulated here with an index set which is a countable set in any type.
Baire theorem: the intersection of two dense Gδ sets is dense.
If a countable family of closed sets cover a dense Gδ set, then the union of their interiors
is dense. Formulated here with ⋃.
If a countable family of closed sets cover a dense Gδ set, then the union of their interiors
is dense. Formulated here with a union over a countable set in any type.
If a countable family of closed sets cover a dense Gδ set, then the union of their interiors
is dense. Formulated here with ⋃₀.
Baire theorem: if countably many closed sets cover the whole space, then their interiors are dense. Formulated here with an index set which is a countable set in any type.
Baire theorem: if countably many closed sets cover the whole space, then their interiors
are dense. Formulated here with ⋃₀.
Baire theorem: if countably many closed sets cover the whole space, then their interiors are dense. Formulated here with an index set which is an encodable type.
One of the most useful consequences of Baire theorem: if a countable union of closed sets covers the space, then one of the sets has nonempty interior.