Documentation

Mathlib.Algebra.Order.GroupWithZero.Lex

Order homomorphisms for products of linearly ordered groups with zero #

This file defines order homomorphisms for products of linearly ordered groups with zero, which is identified with the WithZero of the lexicographic product of the units of the groups.

The product of linearly ordered groups with zero WithZero (αˣ ×ₗ βˣ) is a linearly ordered group with zero itself with natural inclusions but only one projection. One has to work with the lexicographic product of the units αˣ ×ₗ βˣ since otherwise, the plain product αˣ × βˣ would not be linearly ordered.

TODO #

Create the "LinOrdCommGrpWithZero" category.

def toLexMulEquiv (G : Type u_1) (H : Type u_2) [MulOneClass G] [MulOneClass H] :
G × H ≃* Lex (G × H)

toLex as a monoid isomorphism.

Equations
Instances For
    @[simp]
    theorem coe_toLexMulEquiv (G : Type u_1) (H : Type u_2) [MulOneClass G] [MulOneClass H] :
    (toLexMulEquiv G H) = toLex
    @[simp]
    theorem coe_symm_toLexMulEquiv (G : Type u_1) (H : Type u_2) [MulOneClass G] [MulOneClass H] :
    @[simp]
    theorem toEquiv_toLexMulEquiv (G : Type u_1) (H : Type u_2) [MulOneClass G] [MulOneClass H] :
    (toLexMulEquiv G H) = toLex
    @[simp]
    theorem toEquiv_symm_toLexMulEquiv (G : Type u_1) (H : Type u_2) [MulOneClass G] [MulOneClass H] :
    (toLexMulEquiv G H).symm = ofLex
    theorem MonoidWithZeroHom.inl_mono {M₀ : Type u_1} {N₀ : Type u_2} [LinearOrderedCommGroupWithZero M₀] [GroupWithZero N₀] [Preorder N₀] [DecidablePred fun (x : M₀) => x = 0] :
    Monotone (inl M₀ N₀)
    theorem MonoidWithZeroHom.inl_strictMono {M₀ : Type u_1} {N₀ : Type u_2} [LinearOrderedCommGroupWithZero M₀] [GroupWithZero N₀] [PartialOrder N₀] [DecidablePred fun (x : M₀) => x = 0] :
    StrictMono (inl M₀ N₀)
    theorem MonoidWithZeroHom.inr_mono {M₀ : Type u_1} {N₀ : Type u_2} [GroupWithZero M₀] [Preorder M₀] [LinearOrderedCommGroupWithZero N₀] [DecidablePred fun (x : N₀) => x = 0] :
    Monotone (inr M₀ N₀)
    theorem MonoidWithZeroHom.inr_strictMono {M₀ : Type u_1} {N₀ : Type u_2} [GroupWithZero M₀] [PartialOrder M₀] [LinearOrderedCommGroupWithZero N₀] [DecidablePred fun (x : N₀) => x = 0] :
    StrictMono (inr M₀ N₀)
    theorem MonoidWithZeroHom.fst_mono {M₀ : Type u_1} {N₀ : Type u_2} [LinearOrderedCommGroupWithZero M₀] [GroupWithZero N₀] [Preorder N₀] :
    Monotone (fst M₀ N₀)
    theorem MonoidWithZeroHom.snd_mono {M₀ : Type u_1} {N₀ : Type u_2} [GroupWithZero M₀] [Preorder M₀] [LinearOrderedCommGroupWithZero N₀] :
    Monotone (snd M₀ N₀)

    Given linearly ordered groups with zero M, N, the natural inclusion ordered homomorphism from M to WithZero (Mˣ ×ₗ Nˣ), which is the linearly ordered group with zero that can be identified as their product.

    Equations
    Instances For

      Given linearly ordered groups with zero M, N, the natural inclusion ordered homomorphism from N to WithZero (Mˣ ×ₗ Nˣ), which is the linearly ordered group with zero that can be identified as their product.

      Equations
      Instances For

        Given linearly ordered groups with zero M, N, the natural projection ordered homomorphism from WithZero (Mˣ ×ₗ Nˣ) to M, which is the linearly ordered group with zero that can be identified as their product.

        Equations
        Instances For
          theorem LinearOrderedCommGroupWithZero.inl_mul_inr_eq_coe_toLex {α : Type u_1} {β : Type u_2} [LinearOrderedCommGroupWithZero α] [LinearOrderedCommGroupWithZero β] {m : α} {n : β} (hm : m 0) (hn : n 0) :
          (inl α β) m * (inr α β) n = (toLex (Units.mk0 m hm, Units.mk0 n hn))