Documentation

Mathlib.Algebra.Order.Group.Cone

Construct ordered groups from groups with a specified positive cone. #

In this file we provide the structure GroupCone and the predicate IsMaxCone that encode axioms of OrderedCommGroup and LinearOrderedCommGroup in terms of the subset of non-negative elements.

We also provide constructors that convert between cones in groups and the corresponding ordered groups.

class AddGroupConeClass (S : Type u_1) (G : outParam (Type u_2)) [AddCommGroup G] [SetLike S G] extends AddSubmonoidClass S G :

AddGroupConeClass S G says that S is a type of cones in G.

Instances
    class GroupConeClass (S : Type u_1) (G : outParam (Type u_2)) [CommGroup G] [SetLike S G] extends SubmonoidClass S G :

    GroupConeClass S G says that S is a type of cones in G.

    Instances
      structure AddGroupCone (G : Type u_1) [AddCommGroup G] extends AddSubmonoid G :
      Type u_1

      A (positive) cone in an abelian group is a submonoid that does not contain both a and -a for any nonzero a. This is equivalent to being the set of non-negative elements of some order making the group into a partially ordered group.

      Instances For
        structure GroupCone (G : Type u_1) [CommGroup G] extends Submonoid G :
        Type u_1

        A (positive) cone in an abelian group is a submonoid that does not contain both a and a⁻¹ for any non-identity a. This is equivalent to being the set of elements that are at least 1 in some order making the group into a partially ordered group.

        Instances For
          instance GroupCone.instSetLike (G : Type u_1) [CommGroup G] :
          Equations
          Equations
          Equations
          • =
          class IsMaxCone {S : Type u_1} {G : Type u_2} [AddCommGroup G] [SetLike S G] (C : S) :

          Typeclass for maximal additive cones.

          • mem_or_neg_mem : ∀ (a : G), a C -a C
          Instances
            class IsMaxMulCone {S : Type u_1} {G : Type u_2} [CommGroup G] [SetLike S G] (C : S) :

            Typeclass for maximal multiplicative cones.

            Instances

              Construct a cone from the set of elements of a partially ordered abelian group that are at least 1.

              Equations
              Instances For

                Construct a cone from the set of non-negative elements of a partially ordered abelian group.

                Equations
                Instances For
                  @[simp]
                  theorem GroupCone.mem_oneLE {H : Type u_1} [OrderedCommGroup H] {a : H} :
                  @[simp]
                  theorem GroupCone.coe_oneLE {H : Type u_1} [OrderedCommGroup H] :
                  (GroupCone.oneLE H) = {x : H | 1 x}
                  @[simp]
                  theorem AddGroupCone.coe_nonneg {H : Type u_1} [OrderedAddCommGroup H] :
                  (AddGroupCone.nonneg H) = {x : H | 0 x}
                  @[reducible]
                  def OrderedCommGroup.mkOfCone {S : Type u_1} {G : Type u_2} [CommGroup G] [SetLike S G] (C : S) [GroupConeClass S G] :

                  Construct a partially ordered abelian group by designating a cone in an abelian group.

                  Equations
                  Instances For
                    @[reducible]

                    Construct a partially ordered abelian group by designating a cone in an abelian group.

                    Equations
                    Instances For
                      @[reducible]
                      def LinearOrderedCommGroup.mkOfCone {S : Type u_1} {G : Type u_2} [CommGroup G] [SetLike S G] (C : S) [GroupConeClass S G] [IsMaxMulCone C] (dec : DecidablePred fun (x : G) => x C) :

                      Construct a linearly ordered abelian group by designating a maximal cone in an abelian group.

                      Equations
                      Instances For
                        @[reducible]
                        def LinearOrderedAddCommGroup.mkOfCone {S : Type u_1} {G : Type u_2} [AddCommGroup G] [SetLike S G] (C : S) [AddGroupConeClass S G] [IsMaxCone C] (dec : DecidablePred fun (x : G) => x C) :

                        Construct a linearly ordered abelian group by designating a maximal cone in an abelian group.

                        Equations
                        Instances For