Documentation

Mathlib.Topology.Algebra.Order.Group

Topology on a linear ordered commutative group #

In this file we prove that a linear ordered commutative group with order topology is a topological group. We also prove continuity of abs : G → G and provide convenience lemmas like ContinuousAt.abs.

theorem Filter.Tendsto.mabs {G : Type u_1} [TopologicalSpace G] [LinearOrderedCommGroup G] [OrderTopology G] {α : Type u_2} {l : Filter α} {f : αG} {a : G} (h : Tendsto f l (nhds a)) :
Tendsto (fun (x : α) => mabs (f x)) l (nhds (mabs a))
theorem Filter.Tendsto.abs {G : Type u_1} [TopologicalSpace G] [LinearOrderedAddCommGroup G] [OrderTopology G] {α : Type u_2} {l : Filter α} {f : αG} {a : G} (h : Tendsto f l (nhds a)) :
Tendsto (fun (x : α) => |f x|) l (nhds |a|)
theorem Continuous.mabs {G : Type u_1} [TopologicalSpace G] [LinearOrderedCommGroup G] [OrderTopology G] {X : Type u_2} [TopologicalSpace X] {f : XG} (h : Continuous f) :
Continuous fun (x : X) => mabs (f x)
theorem Continuous.abs {G : Type u_1} [TopologicalSpace G] [LinearOrderedAddCommGroup G] [OrderTopology G] {X : Type u_2} [TopologicalSpace X] {f : XG} (h : Continuous f) :
Continuous fun (x : X) => |f x|
theorem ContinuousAt.mabs {G : Type u_1} [TopologicalSpace G] [LinearOrderedCommGroup G] [OrderTopology G] {X : Type u_2} [TopologicalSpace X] {f : XG} {x : X} (h : ContinuousAt f x) :
ContinuousAt (fun (x : X) => mabs (f x)) x
theorem ContinuousAt.abs {G : Type u_1} [TopologicalSpace G] [LinearOrderedAddCommGroup G] [OrderTopology G] {X : Type u_2} [TopologicalSpace X] {f : XG} {x : X} (h : ContinuousAt f x) :
ContinuousAt (fun (x : X) => |f x|) x
theorem ContinuousWithinAt.mabs {G : Type u_1} [TopologicalSpace G] [LinearOrderedCommGroup G] [OrderTopology G] {X : Type u_2} [TopologicalSpace X] {f : XG} {s : Set X} {x : X} (h : ContinuousWithinAt f s x) :
ContinuousWithinAt (fun (x : X) => mabs (f x)) s x
theorem ContinuousWithinAt.abs {G : Type u_1} [TopologicalSpace G] [LinearOrderedAddCommGroup G] [OrderTopology G] {X : Type u_2} [TopologicalSpace X] {f : XG} {s : Set X} {x : X} (h : ContinuousWithinAt f s x) :
ContinuousWithinAt (fun (x : X) => |f x|) s x
theorem ContinuousOn.mabs {G : Type u_1} [TopologicalSpace G] [LinearOrderedCommGroup G] [OrderTopology G] {X : Type u_2} [TopologicalSpace X] {f : XG} {s : Set X} (h : ContinuousOn f s) :
ContinuousOn (fun (x : X) => mabs (f x)) s
theorem ContinuousOn.abs {G : Type u_1} [TopologicalSpace G] [LinearOrderedAddCommGroup G] [OrderTopology G] {X : Type u_2} [TopologicalSpace X] {f : XG} {s : Set X} (h : ContinuousOn f s) :
ContinuousOn (fun (x : X) => |f x|) s
@[deprecated tendsto_abs_nhdsNE_zero (since := "2025-03-18")]

Alias of tendsto_abs_nhdsNE_zero.

theorem denseRange_zpow_iff_surjective {G : Type u_1} [TopologicalSpace G] [LinearOrderedCommGroup G] [OrderTopology G] {a : G} :
(DenseRange fun (x : ) => a ^ x) Function.Surjective fun (x : ) => a ^ x

In a linearly ordered multiplicative group, the integer powers of an element are dense iff they are the whole group.

In a linearly ordered additive group, the integer multiples of an element are dense iff they are the whole group.

In a nontrivial densely linearly ordered commutative group, the integer powers of an element can't be dense.

In a nontrivial densely linearly ordered additive group, the integer multiples of an element can't be dense.