Documentation

Mathlib.RingTheory.OreLocalization.OreSet

(Right) Ore sets #

This defines right Ore sets on arbitrary monoids.

References #

class OreLocalization.OreSet {R : Type u_1} [Monoid R] (S : Submonoid R) :
Type u_1
  • ore_left_cancel : ∀ (r₁ r₂ : R) (s : { x // x S }), s * r₁ = s * r₂s', r₁ * s' = r₂ * s'

    Common factors on the left can be turned into common factors on the right, a weak form of cancellability.

  • oreNum : R{ x // x S }R

    The Ore numerator of a fraction.

  • oreDenom : R{ x // x S }{ x // x S }

    The Ore denominator of a fraction.

  • ore_eq : ∀ (r : R) (s_1 : { x // x S }), r * ↑(OreLocalization.OreSet.oreDenom r s_1) = s_1 * OreLocalization.OreSet.oreNum r s_1

    The Ore condition of a fraction, expressed in terms of oreNum and oreDenom.

A submonoid S of a monoid R is (right) Ore if common factors on the left can be turned into common factors on the right, and if each pair of r : R and s : S admits an Ore numerator v : R and an Ore denominator u : S such that r * u = s * v.

Instances
    theorem OreLocalization.ore_left_cancel {R : Type u_1} [Monoid R] {S : Submonoid R} [OreLocalization.OreSet S] (r₁ : R) (r₂ : R) (s : { x // x S }) (h : s * r₁ = s * r₂) :
    s', r₁ * s' = r₂ * s'

    Common factors on the left can be turned into common factors on the right, a weak form of cancellability.

    def OreLocalization.oreNum {R : Type u_1} [Monoid R] {S : Submonoid R} [OreLocalization.OreSet S] (r : R) (s : { x // x S }) :
    R

    The Ore numerator of a fraction.

    Instances For
      def OreLocalization.oreDenom {R : Type u_1} [Monoid R] {S : Submonoid R} [OreLocalization.OreSet S] (r : R) (s : { x // x S }) :
      { x // x S }

      The Ore denominator of a fraction.

      Instances For
        theorem OreLocalization.ore_eq {R : Type u_1} [Monoid R] {S : Submonoid R} [OreLocalization.OreSet S] (r : R) (s : { x // x S }) :

        The Ore condition of a fraction, expressed in terms of oreNum and oreDenom.

        def OreLocalization.oreCondition {R : Type u_1} [Monoid R] {S : Submonoid R} [OreLocalization.OreSet S] (r : R) (s : { x // x S }) :
        (r' : R) ×' (s' : { x // x S }) ×' r * s' = s * r'

        The Ore condition bundled in a sigma type. This is useful in situations where we want to obtain both witnesses and the condition for a given fraction.

        Instances For

          The trivial submonoid is an Ore set.

          Every submonoid of a commutative monoid is an Ore set.

          def OreLocalization.oreSetOfCancelMonoidWithZero {R : Type u_1} [CancelMonoidWithZero R] {S : Submonoid R} (oreNum : R{ x // x S }R) (oreDenom : R{ x // x S }{ x // x S }) (ore_eq : ∀ (r : R) (s : { x // x S }), r * ↑(oreDenom r s) = s * oreNum r s) :

          Cancellability in monoids with zeros can act as a replacement for the ore_left_cancel condition of an ore set.

          Instances For
            def OreLocalization.oreSetOfNoZeroDivisors {R : Type u_1} [Ring R] [NoZeroDivisors R] {S : Submonoid R} (oreNum : R{ x // x S }R) (oreDenom : R{ x // x S }{ x // x S }) (ore_eq : ∀ (r : R) (s : { x // x S }), r * ↑(oreDenom r s) = s * oreNum r s) :

            In rings without zero divisors, the first (cancellability) condition is always fulfilled, it suffices to give a proof for the Ore condition itself.

            Instances For