(Topological) Schemes and their induced maps #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In topology, and especially descriptive set theory, one often constructs functions (ℕ → β) → α
,
where α is some topological space and β is a discrete space, as an appropriate limit of some map
list β → set α
. We call the latter type of map a "β
-scheme on α
".
This file develops the basic, abstract theory of these schemes and the functions they induce.
Main Definitions #
cantor_scheme.induced_map A
: The aforementioned "limit" of a schemeA : list β → set α
. This is a partial function fromℕ → β
toa
, implemented here as an object of typeΣ s : set (ℕ → β), s → α
. That is,(induced_map A).1
is the domain and(induced_map A).2
is the function.
Implementation Notes #
We consider end-appending to be the fundamental way to build lists (say on β
) inductively,
as this interacts better with the topology on ℕ → β
.
As a result, functions like list.nth
or stream.take
do not have their intended meaning
in this file. See instead pi_nat.res
.
References #
- [Kec95] (Chapters 6-7)
Tags #
scheme, cantor scheme, lusin scheme, approximation.
From a β
-scheme on α
A
, we define a partial function from (ℕ → β)
to α
which sends each infinite sequence x
to an element of the intersection along the
branch corresponding to x
, if it exists.
We call this the map induced by the scheme.
Equations
- cantor_scheme.induced_map A = ⟨λ (x : ℕ → β), (⋂ (n : ℕ), A (pi_nat.res x n)).nonempty, λ (x : ↥(λ (x : ℕ → β), (⋂ (n : ℕ), A (pi_nat.res x n)).nonempty)), set.nonempty.some _⟩
A useful strengthening of being antitone is to require that each set contains the closure of each of its children.
If x
is in the domain of the induced map of a scheme A
,
its image under this map is in each set along the corresponding branch.
A scheme where the children of each set are pairwise disjoint induces an injective map.
A scheme on a metric space has vanishing diameter if diameter approaches 0 along each branch.
Equations
- cantor_scheme.vanishing_diam A = ∀ (x : ℕ → β), filter.tendsto (λ (n : ℕ), emetric.diam (A (pi_nat.res x n))) filter.at_top (nhds 0)
A scheme with vanishing diameter along each branch induces a continuous map.
A scheme on a complete space with vanishing diameter such that each set contains the closure of its children induces a total map.