Documentation

Mathlib.Topology.Algebra.Group.GroupTopology

Lattice of group topologies #

We define a type class GroupTopology α which endows a group α with a topology such that all group operations are continuous.

Group topologies on a fixed group α are ordered, by reverse inclusion. They form a complete lattice, with the discrete topology and the indiscrete topology.

Any function f : α → β induces coinduced f : TopologicalSpace α → GroupTopology β.

The additive version AddGroupTopology α and corresponding results are provided as well.

structure GroupTopology (α : Type u) [Group α] extends TopologicalSpace α, IsTopologicalGroup α :

A group topology on a group α is a topology for which multiplication and inversion are continuous.

Instances For
    structure AddGroupTopology (α : Type u) [AddGroup α] extends TopologicalSpace α, IsTopologicalAddGroup α :

    An additive group topology on an additive group α is a topology for which addition and negation are continuous.

    Instances For
      theorem GroupTopology.continuous_mul' {α : Type u} [Group α] (g : GroupTopology α) :
      Continuous fun (p : α × α) => p.1 * p.2

      A version of the global continuous_mul suitable for dot notation.

      theorem AddGroupTopology.continuous_add' {α : Type u} [AddGroup α] (g : AddGroupTopology α) :
      Continuous fun (p : α × α) => p.1 + p.2

      A version of the global continuous_add suitable for dot notation.

      A version of the global continuous_inv suitable for dot notation.

      A version of the global continuous_neg suitable for dot notation.

      The ordering on group topologies on the group γ. t ≤ s if every set open in s is also open in t (t is finer than s).

      Equations

      The ordering on group topologies on the group γ. t ≤ s if every set open in s is also open in t (t is finer than s).

      Equations
      instance GroupTopology.instTop {α : Type u} [Group α] :
      Equations
      Equations
      instance GroupTopology.instBot {α : Type u} [Group α] :
      Equations
      Equations
      instance GroupTopology.instMin {α : Type u} [Group α] :
      Equations
      Equations

      Infimum of a collection of group topologies.

      Equations

      Infimum of a collection of additive group topologies

      Equations
      @[simp]
      theorem GroupTopology.toTopologicalSpace_iInf {α : Type u} [Group α] {ι : Sort u_1} (s : ιGroupTopology α) :
      (⨅ (i : ι), s i).toTopologicalSpace = ⨅ (i : ι), (s i).toTopologicalSpace
      @[simp]
      theorem AddGroupTopology.toTopologicalSpace_iInf {α : Type u} [AddGroup α] {ι : Sort u_1} (s : ιAddGroupTopology α) :
      (⨅ (i : ι), s i).toTopologicalSpace = ⨅ (i : ι), (s i).toTopologicalSpace

      Group topologies on γ form a complete lattice, with the discrete topology and the indiscrete topology.

      The infimum of a collection of group topologies is the topology generated by all their open sets (which is a group topology).

      The supremum of two group topologies s and t is the infimum of the family of all group topologies contained in the intersection of s and t.

      Equations

      Group topologies on γ form a complete lattice, with the discrete topology and the indiscrete topology.

      The infimum of a collection of group topologies is the topology generated by all their open sets (which is a group topology).

      The supremum of two group topologies s and t is the infimum of the family of all group topologies contained in the intersection of s and t.

      Equations
      def GroupTopology.coinduced {α : Type u_1} {β : Type u_2} [t : TopologicalSpace α] [Group β] (f : αβ) :

      Given f : α → β and a topology on α, the coinduced group topology on β is the finest topology such that f is continuous and β is a topological group.

      Equations
      Instances For
        def AddGroupTopology.coinduced {α : Type u_1} {β : Type u_2} [t : TopologicalSpace α] [AddGroup β] (f : αβ) :

        Given f : α → β and a topology on α, the coinduced additive group topology on β is the finest topology such that f is continuous and β is a topological additive group.

        Equations
        Instances For
          theorem GroupTopology.coinduced_continuous {α : Type u_1} {β : Type u_2} [t : TopologicalSpace α] [Group β] (f : αβ) :
          theorem AddGroupTopology.coinduced_continuous {α : Type u_1} {β : Type u_2} [t : TopologicalSpace α] [AddGroup β] (f : αβ) :