Documentation

Mathlib.Topology.Algebra.IsOpenUnits

Topological monoids with open units #

We say that a topological monoid M has open units (IsOpenUnits) if is open in M and has the subspace topology (i.e. inverse is continuous).

Typical examples include monoids with discrete topology, topological groups (or fields), and rings R equipped with the I-adic topology where I ≤ J(R) (IsOpenUnits.of_isAdic).

A non-example is 𝔸ₖ, because the topology on ideles is not the induced topology from adeles.

This condition is necessary and sufficient for U(R) to be an open subspace of X(R) for all affine scheme X over R and all affine open subscheme U ⊆ X.

class IsOpenUnits (M : Type u_1) [Monoid M] [TopologicalSpace M] :

We say that a topological monoid M has open units if is open in M and has the subspace topology (i.e. inverse is continuous).

Typical examples include monoids with discrete topology, topological groups (or fields), and rings R equipped with the I-adic topology where I ≤ J(R).

Instances
    theorem IsOpenUnits.of_isAdic {R : Type u_1} [CommRing R] [TopologicalSpace R] [IsTopologicalRing R] {I : Ideal R} (hR : IsAdic I) (hI : I .jacobson) :

    If R has the I-adic topology where I is contained in the jacobson radical (e.g. when R is complete or local), then is an open subspace of R.