Documentation

Mathlib.GroupTheory.MonoidLocalization.Order

Ordered structures on localizations of commutative monoids #

theorem AddLocalization.le.proof_1 {α : Type u_1} [OrderedCancelAddCommMonoid α] {s : AddSubmonoid α} {a₁ : α} {b₁ : α} {a₂ : s} {b₂ : s} {c₁ : α} {d₁ : α} {c₂ : s} {d₂ : s} (hab : (AddLocalization.r s) (a₁, a₂) (b₁, b₂)) (hcd : (AddLocalization.r s) (c₁, c₂) (d₁, d₂)) :
(fun (a₁ : α) (a₂ : s) (b₁ : α) (b₂ : s) => b₂ + a₁ a₂ + b₁) a₁ a₂ c₁ c₂ = (fun (a₁ : α) (a₂ : s) (b₁ : α) (b₂ : s) => b₂ + a₁ a₂ + b₁) b₁ b₂ d₁ d₂
Equations
  • AddLocalization.le = { le := fun (a b : AddLocalization s) => a.liftOn₂ b (fun (a₁ : α) (a₂ : s) (b₁ : α) (b₂ : s) => b₂ + a₁ a₂ + b₁) }
instance Localization.le {α : Type u_1} [OrderedCancelCommMonoid α] {s : Submonoid α} :
Equations
  • Localization.le = { le := fun (a b : Localization s) => a.liftOn₂ b (fun (a₁ : α) (a₂ : s) (b₁ : α) (b₂ : s) => b₂ * a₁ a₂ * b₁) }
theorem AddLocalization.lt.proof_1 {α : Type u_1} [OrderedCancelAddCommMonoid α] {s : AddSubmonoid α} {a₁ : α} {b₁ : α} {a₂ : s} {b₂ : s} {c₁ : α} {d₁ : α} {c₂ : s} {d₂ : s} (hab : (AddLocalization.r s) (a₁, a₂) (b₁, b₂)) (hcd : (AddLocalization.r s) (c₁, c₂) (d₁, d₂)) :
(fun (a₁ : α) (a₂ : s) (b₁ : α) (b₂ : s) => b₂ + a₁ < a₂ + b₁) a₁ a₂ c₁ c₂ = (fun (a₁ : α) (a₂ : s) (b₁ : α) (b₂ : s) => b₂ + a₁ < a₂ + b₁) b₁ b₂ d₁ d₂
Equations
  • AddLocalization.lt = { lt := fun (a b : AddLocalization s) => a.liftOn₂ b (fun (a₁ : α) (a₂ : s) (b₁ : α) (b₂ : s) => b₂ + a₁ < a₂ + b₁) }
instance Localization.lt {α : Type u_1} [OrderedCancelCommMonoid α] {s : Submonoid α} :
Equations
  • Localization.lt = { lt := fun (a b : Localization s) => a.liftOn₂ b (fun (a₁ : α) (a₂ : s) (b₁ : α) (b₂ : s) => b₂ * a₁ < a₂ * b₁) }
theorem AddLocalization.mk_le_mk {α : Type u_1} [OrderedCancelAddCommMonoid α] {s : AddSubmonoid α} {a₁ : α} {b₁ : α} {a₂ : s} {b₂ : s} :
AddLocalization.mk a₁ a₂ AddLocalization.mk b₁ b₂ b₂ + a₁ a₂ + b₁
theorem Localization.mk_le_mk {α : Type u_1} [OrderedCancelCommMonoid α] {s : Submonoid α} {a₁ : α} {b₁ : α} {a₂ : s} {b₂ : s} :
Localization.mk a₁ a₂ Localization.mk b₁ b₂ b₂ * a₁ a₂ * b₁
theorem AddLocalization.mk_lt_mk {α : Type u_1} [OrderedCancelAddCommMonoid α] {s : AddSubmonoid α} {a₁ : α} {b₁ : α} {a₂ : s} {b₂ : s} :
AddLocalization.mk a₁ a₂ < AddLocalization.mk b₁ b₂ b₂ + a₁ < a₂ + b₁
theorem Localization.mk_lt_mk {α : Type u_1} [OrderedCancelCommMonoid α] {s : Submonoid α} {a₁ : α} {b₁ : α} {a₂ : s} {b₂ : s} :
Localization.mk a₁ a₂ < Localization.mk b₁ b₂ b₂ * a₁ < a₂ * b₁
Equations
Equations
Equations
instance AddLocalization.decidableLE {α : Type u_1} [OrderedCancelAddCommMonoid α] {s : AddSubmonoid α} [DecidableRel fun (x x_1 : α) => x x_1] :
DecidableRel fun (x x_1 : AddLocalization s) => x x_1
Equations
  • a.decidableLE b = a.recOnSubsingleton₂ b fun (x x_1 : α) (x_2 x_3 : s) => decidable_of_iff' (x_3 + x x_2 + x_1)
theorem AddLocalization.decidableLE.proof_1 {α : Type u_1} [OrderedCancelAddCommMonoid α] {s : AddSubmonoid α} (a : α) (c : α) (b : s) (d : s) :
instance Localization.decidableLE {α : Type u_1} [OrderedCancelCommMonoid α] {s : Submonoid α} [DecidableRel fun (x x_1 : α) => x x_1] :
DecidableRel fun (x x_1 : Localization s) => x x_1
Equations
  • a.decidableLE b = a.recOnSubsingleton₂ b fun (x x_1 : α) (x_2 x_3 : s) => decidable_of_iff' (x_3 * x x_2 * x_1)
theorem AddLocalization.decidableLT.proof_1 {α : Type u_1} [OrderedCancelAddCommMonoid α] {s : AddSubmonoid α} (a : α) (c : α) (b : s) (d : s) :
instance AddLocalization.decidableLT {α : Type u_1} [OrderedCancelAddCommMonoid α] {s : AddSubmonoid α} [DecidableRel fun (x x_1 : α) => x < x_1] :
DecidableRel fun (x x_1 : AddLocalization s) => x < x_1
Equations
  • a.decidableLT b = a.recOnSubsingleton₂ b fun (x x_1 : α) (x_2 x_3 : s) => decidable_of_iff' (x_3 + x < x_2 + x_1)
instance Localization.decidableLT {α : Type u_1} [OrderedCancelCommMonoid α] {s : Submonoid α} [DecidableRel fun (x x_1 : α) => x < x_1] :
DecidableRel fun (x x_1 : Localization s) => x < x_1
Equations
  • a.decidableLT b = a.recOnSubsingleton₂ b fun (x x_1 : α) (x_2 x_3 : s) => decidable_of_iff' (x_3 * x < x_2 * x_1)
theorem AddLocalization.mkOrderEmbedding.proof_2 {α : Type u_1} [OrderedCancelAddCommMonoid α] {s : AddSubmonoid α} (b : s) {a : α} {b : α} :

An ordered cancellative monoid injects into its localization by sending a to a - b.

Equations
Instances For
    @[simp]

    An ordered cancellative monoid injects into its localization by sending a to a / b.

    Equations
    Instances For
      Equations
      • One or more equations did not get rendered due to their size.
      Equations
      • One or more equations did not get rendered due to their size.