Documentation

Mathlib.Analysis.Normed.Ring.IsPowMulFaithful

Equivalent power-multiplicative norms #

In this file, we prove [BGR, Proposition 3.1.5/1][bosch-guntzer-remmert]: if R is a normed commutative ring and f₁ and f₂ are two power-multiplicative R-algebra norms on S, then if f₁ and f₂ are equivalent on every subring R[y] for y : S, it follows that f₁ = f₂.

Main Results #

References #

Tags #

norm, equivalent, power-multiplicative

theorem contraction_of_isPowMul_of_boundedWrt {F : Type u_1} {α : outParam (Type u_2)} [Ring α] [FunLike F α ] [RingSeminormClass F α ] {β : Type u_3} [Ring β] (nα : F) {nβ : β} (hβ : IsPowMul ) {f : α →+* β} (hf : RingHom.IsBoundedWrt (⇑) f) (x : α) :
(f x) x

If f : α →+* β is bounded with respect to a ring seminorm on α and a power-multiplicative function nβ : β → ℝ, then ∀ x : α, nβ (f x) ≤ nα x.

theorem contraction_of_isPowMul {α : Type u_1} {β : Type u_2} [SeminormedRing α] [SeminormedRing β] (hβ : IsPowMul norm) {f : α →+* β} (hf : f.IsBounded) (x : α) :

Given a bounded f : α →+* β between seminormed rings, is the seminorm on β is power-multiplicative, then f is a contraction.

theorem eq_seminorms {F : Type u_1} {α : outParam (Type u_2)} [Ring α] [FunLike F α ] [RingSeminormClass F α ] {f : F} {g : F} (hfpm : IsPowMul f) (hgpm : IsPowMul g) (hfg : ∃ (r : ) (_ : 0 < r), ∀ (a : α), f a r * g a) (hgf : ∃ (r : ) (_ : 0 < r), ∀ (a : α), g a r * f a) :
f = g

Given two power-multiplicative ring seminorms f, g on α, if f is bounded by a positive multiple of g and vice versa, then f = g.

theorem eq_of_powMul_faithful {R : Type u_1} {S : Type u_2} [NormedCommRing R] [CommRing S] [Algebra R S] (f₁ : AlgebraNorm R S) (hf₁_pm : IsPowMul f₁) (f₂ : AlgebraNorm R S) (hf₂_pm : IsPowMul f₂) (h_eq : ∀ (y : S), ∃ (C₁ : ) (C₂ : ) (_ : 0 < C₁) (_ : 0 < C₂), ∀ (x : (Algebra.adjoin R {y})), f₁ x C₁ * f₂ x f₂ x C₂ * f₁ x) :
f₁ = f₂

If R is a normed commutative ring and f₁ and f₂ are two power-multiplicative R-algebra norms on S, then if f₁ and f₂ are equivalent on every subring R[y] for y : S, it follows that f₁ = f₂ [BGR, Proposition 3.1.5/1][bosch-guntzer-remmert].