Flows and invariant sets #
This file defines a flow on a topological space α by a topological
monoid τ as a continuous monoid-action of τ on α. Anticipating the
cases where τ is one of ℕ, ℤ, ℝ⁺, or ℝ, we use additive
notation for the monoids, though the definition does not require
commutativity.
A subset s of α is invariant under a family of maps ϕₜ : α → α
if ϕₜ s ⊆ s for all t. In many cases ϕ will be a flow on
α. For the cases where ϕ is a flow by an ordered (additive,
commutative) monoid, we additionally define forward invariance, where
t ranges over those elements which are nonnegative.
Additionally, we define such constructions as the (forward) orbit, a semiconjugacy between flows, a factor of a flow, the restriction of a flow onto an invariant subset, and the time-reversal of a flow by a group.
Invariant sets #
A set s ⊆ α is invariant under ϕ : τ → α → α if ϕ t s ⊆ s for all t in τ.
Equations
- IsInvariant ϕ s = ∀ (t : τ), Set.MapsTo (ϕ t) s s
Instances For
A set s ⊆ α is forward-invariant under ϕ : τ → α → α if ϕ t s ⊆ s for all t ≥ 0.
Equations
- IsForwardInvariant ϕ s = ∀ ⦃t : τ⦄, 0 ≤ t → Set.MapsTo (ϕ t) s s
Instances For
Alias of IsForwardInvariant.
A set s ⊆ α is forward-invariant under ϕ : τ → α → α if ϕ t s ⊆ s for all t ≥ 0.
Equations
Instances For
Alias of IsInvariant.isForwardInvariant.
If τ is a CanonicallyOrderedAdd monoid (e.g., ℕ or ℝ≥0), then the notions
IsForwardInvariant and IsInvariant are equivalent.
Alias of IsForwardInvariant.isInvariant.
If τ is a CanonicallyOrderedAdd monoid (e.g., ℕ or ℝ≥0), then the notions
IsForwardInvariant and IsInvariant are equivalent.
If τ is a CanonicallyOrderedAdd monoid (e.g., ℕ or ℝ≥0), then the notions
IsForwardInvariant and IsInvariant are equivalent.
Alias of isForwardInvariant_iff_isInvariant.
If τ is a CanonicallyOrderedAdd monoid (e.g., ℕ or ℝ≥0), then the notions
IsForwardInvariant and IsInvariant are equivalent.
Flows #
A flow on a topological space α by an additive topological
monoid τ is a continuous monoid action of τ on α.
- toFun : τ → α → α
The map
τ → α → αunderlying a flow ofτonα. - cont' : Continuous (Function.uncurry self.toFun)
Instances For
Equations
- Flow.instCoeFunForallForall = { coe := Flow.toFun }
Alias of Flow.continuous.
Iterations of a continuous function from a topological space α
to itself defines a semiflow by ℕ on α.
Equations
Instances For
Restriction of a flow onto an invariant set.
Equations
Instances For
Convert a flow to an additive monoid action.
Equations
- ϕ.toAddAction = { vadd := ϕ.toFun, zero_vadd := ⋯, add_vadd := ⋯ }
Instances For
Restrict a flow by τ to a flow by an additive submonoid of τ.
Equations
- ϕ.restrictAddSubmonoid S = { toFun := fun (t : ↥S) (x : α) => ϕ.toFun (↑t) x, cont' := ⋯, map_add' := ⋯, map_zero' := ⋯ }
Instances For
The orbit of a point under a flow.
Equations
- ϕ.orbit x = AddAction.orbit τ x
Instances For
The orbit of a point under a flow ϕ is invariant under ϕ.
Restrict a flow by τ to a flow by the additive submonoid of nonnegative elements of τ.
Equations
Instances For
The forward orbit of a point under a flow.
Equations
- ϕ.forwardOrbit x = ϕ.restrictNonneg.orbit x
Instances For
The forward orbit of a point under a flow ϕ is forward-invariant under ϕ.
The forward orbit of a point x is contained in the orbit of x.
Given flows ϕ by τ on α and ψ by τ on β, a function π : α → β is called a
semiconjugacy from ϕ to ψ if π is continuous and surjective, and π ∘ (ϕ t) = (ψ t) ∘ π for
all t : τ.
- cont : Continuous π
- surj : Function.Surjective π
- semiconj (t : τ) : Function.Semiconj π (ϕ.toFun t) (ψ.toFun t)
Instances For
The composition of semiconjugacies is a semiconjugacy.
The identity is a semiconjugacy from ϕ to ψ if and only if ϕ and ψ are equal.
A flow ψ is called a factor of ϕ if there exists a semiconjugacy from ϕ to ψ.
Equations
- ψ.IsFactorOf ϕ = ∃ (π : α → β), Flow.IsSemiconjugacy π ϕ ψ
Instances For
Transitivity of factors of flows.
Every flow is a factor of itself.
The time-reversal of a flow ϕ by a (commutative, additive) group
is defined ϕ.reverse t x = ϕ (-t) x.
Equations
Instances For
The map ϕ t as a homeomorphism.