Documentation

Mathlib.Algebra.Order.Group.Cyclic

Cyclic linearly ordered groups #

This file contains basic results about cyclic linearly ordered groups and cyclic subgroups of linearly ordered groups.

The definitions LinearOrderedCommGroup.Subgroup.genLTOne (resp. LinearOrderedCommGroup.genLTOone) yields a generator of a non-trivial subgroup of a linearly ordered commutative group with (resp. of a non-trivial linearly ordered commutative group) that is strictly less than 1. The corresponding additive definitions are also provided.

noncomputable def LinearOrderedCommGroup.Subgroup.genLTOne {G : Type u_1} [CommGroup G] [LinearOrder G] [IsOrderedMonoid G] (H : Subgroup G) [Nontrivial H] [hH : IsCyclic H] :
G

Given a subgroup of a cyclic linearly ordered commutative group, this is a generator of the subgroup that is < 1.

Equations
Instances For

    Given an additive subgroup of an additive cyclic linearly ordered commutative group, this is a negative generator of the subgroup.

    Equations
    Instances For
      theorem LinearOrderedCommGroup.Subgroup.genLTOne_unique_of_zpowers_eq {G : Type u_1} [CommGroup G] [LinearOrder G] [IsOrderedMonoid G] {g1 g2 : G} (hg1 : g1 < 1) (hg2 : g2 < 1) (h : Subgroup.zpowers g1 = Subgroup.zpowers g2) :
      g1 = g2

      Given a cyclic linearly ordered commutative group, this is a generator that is < 1.

      Equations
      Instances For

        Given an additive cyclic linearly ordered commutative group, this is a negative generator of it.

        Equations
        Instances For