mathlib3 documentation

dynamics.ergodic.conservative

Conservative systems #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

In this file we define f : α → α to be a conservative system w.r.t a measure μ if f is non-singular (measure_theory.quasi_measure_preserving) and for every measurable set s of positive measure at least one point x ∈ s returns back to s after some number of iterations of f. There are several properties that look like they are stronger than this one but actually follow from it:

We also prove the topological Poincaré recurrence theorem measure_theory.conservative.ae_frequently_mem_of_mem_nhds. Let f : α → α be a conservative dynamical system on a topological space with second countable topology and measurable open sets. Then almost every point x : α is recurrent: it visits every neighborhood s ∈ 𝓝 x infinitely many times.

Tags #

conservative dynamical system, Poincare recurrence theorem

structure measure_theory.conservative {α : Type u_2} [measurable_space α] (f : α α) (μ : measure_theory.measure α . "volume_tac") :
Prop

We say that a non-singular (measure_theory.quasi_measure_preserving) self-map is conservative if for any measurable set s of positive measure there exists x ∈ s such that x returns back to s under some iteration of f.

@[protected]

A self-map preserving a finite measure is conservative.

@[protected]

The identity map is conservative w.r.t. any measure.

If f is a conservative map and s is a measurable set of nonzero measure, then for infinitely many values of m a positive measure of points x ∈ s returns back to s after m iterations of f.

theorem measure_theory.conservative.exists_gt_measure_inter_ne_zero {α : Type u_2} [measurable_space α] {f : α α} {s : set α} {μ : measure_theory.measure α} (hf : measure_theory.conservative f μ) (hs : measurable_set s) (h0 : μ s 0) (N : ) :
(m : ) (H : m > N), μ (s f^[m] ⁻¹' s) 0

If f is a conservative map and s is a measurable set of nonzero measure, then for an arbitrarily large m a positive measure of points x ∈ s returns back to s after m iterations of f.

theorem measure_theory.conservative.measure_mem_forall_ge_image_not_mem_eq_zero {α : Type u_2} [measurable_space α] {f : α α} {s : set α} {μ : measure_theory.measure α} (hf : measure_theory.conservative f μ) (hs : measurable_set s) (n : ) :
μ {x ∈ s | (m : ), m n f^[m] x s} = 0

Poincaré recurrence theorem: given a conservative map f and a measurable set s, the set of points x ∈ s such that x does not return to s after ≥ n iterations has measure zero.

Poincaré recurrence theorem: given a conservative map f and a measurable set s, almost every point x ∈ s returns back to s infinitely many times.

Poincaré recurrence theorem: if f is a conservative dynamical system and s is a measurable set, then for μ-a.e. x, if the orbit of x visits s at least once, then it visits s infinitely many times.

If f is a conservative self-map and s is a measurable set of positive measure, then μ.ae-frequently we have x ∈ s and s returns to s under infinitely many iterations of f.

Poincaré recurrence theorem. Let f : α → α be a conservative dynamical system on a topological space with second countable topology and measurable open sets. Then almost every point x : α is recurrent: it visits every neighborhood s ∈ 𝓝 x infinitely many times.

@[protected]

Iteration of a conservative system is a conservative system.