doc-next-gen

Mathlib.RingTheory.TwoSidedIdeal.Basic

Module docstring

{"# Two Sided Ideals

In this file, for any Ring R, we reinterpret I : RingCon R as a two-sided-ideal of a ring.

Main definitions and results

  • TwoSidedIdeal: For any NonUnitalNonAssocRing R, TwoSidedIdeal R is a wrapper around RingCon R.
  • TwoSidedIdeal.setLike: Every I : TwoSidedIdeal R can be interpreted as a set of R where x ∈ I if and only if I.ringCon x 0.
  • TwoSidedIdeal.addCommGroup: Every I : TwoSidedIdeal R is an abelian group.

"}

TwoSidedIdeal structure
(R : Type*) [NonUnitalNonAssocRing R]
Full source
/--
A two-sided ideal of a ring `R` is a subset of `R` that contains `0` and is closed under addition,
negation, and absorbs multiplication on both sides.
-/
structure TwoSidedIdeal (R : Type*) [NonUnitalNonAssocRing R] where
  /-- every two-sided-ideal is induced by a congruence relation on the ring. -/
  ringCon : RingCon R
Two-sided ideal of a non-unital non-associative ring
Informal description
A two-sided ideal of a non-unital non-associative ring \( R \) is a subset \( I \subseteq R \) that satisfies the following properties: 1. Contains the zero element: \( 0 \in I \). 2. Closed under addition: for any \( x, y \in I \), \( x + y \in I \). 3. Closed under negation: for any \( x \in I \), \( -x \in I \). 4. Absorbs multiplication on both sides: for any \( r \in R \) and \( x \in I \), both \( r \cdot x \in I \) and \( x \cdot r \in I \).
TwoSidedIdeal.setLike instance
: SetLike (TwoSidedIdeal R) R
Full source
instance setLike : SetLike (TwoSidedIdeal R) R where
  coe t := {r | t.ringCon r 0}
  coe_injective'  := by
    rintro ⟨t₁⟩ ⟨t₂⟩ (h : {x | _} = {x | _})
    congr 1
    refine RingCon.ext fun a b ↦ ⟨fun H ↦ ?_, fun H ↦ ?_⟩
    · have H' : a - b ∈ {x | t₁ x 0} := sub_self b ▸ t₁.sub H (t₁.refl b)
      rw [h] at H'
      convert t₂.add H' (t₂.refl b) using 1 <;> abel
    · have H' : a - b ∈ {x | t₂ x 0} := sub_self b ▸ t₂.sub H (t₂.refl b)
      rw [← h] at H'
      convert t₁.add H' (t₁.refl b) using 1 <;> abel
Set-like Structure of Two-sided Ideals
Informal description
For any non-unital non-associative ring $R$, the type of two-sided ideals of $R$ can be interpreted as a set-like structure, where membership $x \in I$ for $x \in R$ and $I$ a two-sided ideal is defined by the congruence relation $I.\text{ringCon}(x, 0)$.
TwoSidedIdeal.mem_iff theorem
(x : R) : x ∈ I ↔ I.ringCon x 0
Full source
lemma mem_iff (x : R) : x ∈ Ix ∈ I ↔ I.ringCon x 0 := Iff.rfl
Membership Criterion for Two-Sided Ideals via Ring Congruence
Informal description
For any element $x$ in a non-unital non-associative ring $R$ and any two-sided ideal $I$ of $R$, the membership $x \in I$ holds if and only if the ring congruence relation $I.\text{ringCon}$ relates $x$ to $0$.
TwoSidedIdeal.mem_mk theorem
{x : R} {c : RingCon R} : x ∈ mk c ↔ c x 0
Full source
@[simp]
lemma mem_mk {x : R} {c : RingCon R} : x ∈ mk cx ∈ mk c ↔ c x 0 := Iff.rfl
Membership Criterion for Two-Sided Ideal via Congruence Relation
Informal description
For any element $x$ in a ring $R$ and any ring congruence relation $c$ on $R$, the element $x$ belongs to the two-sided ideal generated by $c$ if and only if $x$ is congruent to $0$ under $c$, i.e., $c(x, 0)$ holds.
TwoSidedIdeal.coe_mk theorem
{c : RingCon R} : (mk c : Set R) = {x | c x 0}
Full source
@[simp, norm_cast]
lemma coe_mk {c : RingCon R} : (mk c : Set R) = {x | c x 0} := rfl
Characterization of Two-Sided Ideal via Congruence Relation
Informal description
For any ring congruence relation $c$ on a non-unital non-associative ring $R$, the underlying set of the two-sided ideal generated by $c$ is equal to the set $\{x \in R \mid c(x, 0)\}$.
TwoSidedIdeal.rel_iff theorem
(x y : R) : I.ringCon x y ↔ x - y ∈ I
Full source
lemma rel_iff (x y : R) : I.ringCon x y ↔ x - y ∈ I := by
  rw [mem_iff]
  constructor
  · intro h; convert I.ringCon.sub h (I.ringCon.refl y); abel
  · intro h; convert I.ringCon.add h (I.ringCon.refl y) <;> abel
Congruence Relation Characterization via Ideal Membership: $x \sim y \leftrightarrow x - y \in I$
Informal description
For any elements $x$ and $y$ in a non-unital non-associative ring $R$ and any two-sided ideal $I$ of $R$, the congruence relation $I.\text{ringCon}(x, y)$ holds if and only if the difference $x - y$ belongs to $I$.
TwoSidedIdeal.coeOrderEmbedding definition
: TwoSidedIdeal R ↪o Set R
Full source
/--
the coercion from two-sided-ideals to sets is an order embedding
-/
@[simps]
def coeOrderEmbedding : TwoSidedIdealTwoSidedIdeal R ↪o Set R where
  toFun := SetLike.coe
  inj' := SetLike.coe_injective
  map_rel_iff' {I J} := ⟨fun (h : (I : Set R) ⊆ (J : Set R)) _ h' ↦ h h', fun h _ h' ↦ h h'⟩
Order embedding from two-sided ideals to sets
Informal description
The function that coerces a two-sided ideal $I$ of a non-unital non-associative ring $R$ to its underlying set is an order embedding. This means it is an injective function that preserves and reflects the order relation, i.e., for any two-sided ideals $I$ and $J$, $I \leq J$ if and only if the underlying set of $I$ is a subset of the underlying set of $J$.
TwoSidedIdeal.le_iff theorem
{I J : TwoSidedIdeal R} : I ≤ J ↔ (I : Set R) ⊆ (J : Set R)
Full source
lemma le_iff {I J : TwoSidedIdeal R} : I ≤ J ↔ (I : Set R) ⊆ (J : Set R) := Iff.rfl
Order Relation on Two-Sided Ideals via Subset Inclusion
Informal description
For any two-sided ideals $I$ and $J$ of a non-unital non-associative ring $R$, the inequality $I \leq J$ holds if and only if $I$ is a subset of $J$ when viewed as subsets of $R$.
TwoSidedIdeal.orderIsoRingCon definition
: TwoSidedIdeal R ≃o RingCon R
Full source
/-- Two-sided-ideals corresponds to congruence relations on a ring. -/
@[simps apply symm_apply]
def orderIsoRingCon : TwoSidedIdealTwoSidedIdeal R ≃o RingCon R where
  toFun := TwoSidedIdeal.ringCon
  invFun := .mk
  left_inv _ := rfl
  right_inv _ := rfl
  map_rel_iff' {I J} := Iff.symm <| le_iff.trans ⟨fun h x y r => by rw [rel_iff] at r ⊢; exact h r,
    fun h x hx => by rw [SetLike.mem_coe, mem_iff] at hx ⊢; exact h hx⟩
Order isomorphism between two-sided ideals and ring congruence relations
Informal description
The order isomorphism between the type of two-sided ideals of a non-unital non-associative ring \( R \) and the type of ring congruence relations on \( R \). Specifically, it maps each two-sided ideal \( I \) to its associated ring congruence relation \( \text{ringCon}(I) \), and vice versa, preserving the order structure in both directions.
TwoSidedIdeal.ringCon_injective theorem
: Function.Injective (TwoSidedIdeal.ringCon (R := R))
Full source
lemma ringCon_injective : Function.Injective (TwoSidedIdeal.ringCon (R := R)) := by
  rintro ⟨x⟩ ⟨y⟩ rfl; rfl
Injectivity of the Ideal-to-Congruence Relation Map
Informal description
The function mapping a two-sided ideal $I$ of a non-unital non-associative ring $R$ to its associated ring congruence relation is injective. That is, if two ideals $I$ and $J$ induce the same ring congruence relation, then $I = J$.
TwoSidedIdeal.ringCon_le_iff theorem
{I J : TwoSidedIdeal R} : I ≤ J ↔ I.ringCon ≤ J.ringCon
Full source
lemma ringCon_le_iff {I J : TwoSidedIdeal R} : I ≤ J ↔ I.ringCon ≤ J.ringCon :=
  orderIsoRingCon.map_rel_iff.symm
Order Correspondence Between Two-Sided Ideals and Their Congruence Relations
Informal description
For any two-sided ideals $I$ and $J$ of a non-unital non-associative ring $R$, the inequality $I \leq J$ holds if and only if the associated ring congruence relation of $I$ is contained in that of $J$, i.e., $I.\text{ringCon} \leq J.\text{ringCon}$.
TwoSidedIdeal.ext theorem
{I J : TwoSidedIdeal R} (h : ∀ x, x ∈ I ↔ x ∈ J) : I = J
Full source
@[ext]
lemma ext {I J : TwoSidedIdeal R} (h : ∀ x, x ∈ Ix ∈ I ↔ x ∈ J) : I = J :=
  coeOrderEmbedding.injective (Set.ext h)
Extensionality of Two-Sided Ideals: $I = J \iff \forall x, x \in I \leftrightarrow x \in J$
Informal description
For any two-sided ideals $I$ and $J$ of a non-unital non-associative ring $R$, if $x \in I$ if and only if $x \in J$ for all $x \in R$, then $I = J$.
TwoSidedIdeal.lt_iff theorem
(I J : TwoSidedIdeal R) : I < J ↔ (I : Set R) ⊂ (J : Set R)
Full source
lemma lt_iff (I J : TwoSidedIdeal R) : I < J ↔ (I : Set R) ⊂ (J : Set R) := by
  rw [lt_iff_le_and_ne, Set.ssubset_iff_subset_ne, le_iff]
  simp
Characterization of Strict Ideal Inclusion via Strict Subset Relation
Informal description
For any two-sided ideals $I$ and $J$ of a non-unital non-associative ring $R$, the strict inequality $I < J$ holds if and only if $I$ is a strict subset of $J$ when viewed as subsets of $R$.
TwoSidedIdeal.zero_mem theorem
: 0 ∈ I
Full source
@[simp]
lemma zero_mem : 0 ∈ I := I.ringCon.refl 0
Zero Element Belongs to Two-Sided Ideal
Informal description
For any two-sided ideal $I$ of a non-unital non-associative ring $R$, the zero element $0$ is contained in $I$.
TwoSidedIdeal.add_mem theorem
{x y} (hx : x ∈ I) (hy : y ∈ I) : x + y ∈ I
Full source
lemma add_mem {x y} (hx : x ∈ I) (hy : y ∈ I) : x + y ∈ I := by simpa using I.ringCon.add hx hy
Closure of Two-Sided Ideal Under Addition
Informal description
For any two-sided ideal $I$ of a non-unital non-associative ring $R$, if $x \in I$ and $y \in I$, then $x + y \in I$.
TwoSidedIdeal.neg_mem theorem
{x} (hx : x ∈ I) : -x ∈ I
Full source
lemma neg_mem {x} (hx : x ∈ I) : -x ∈ I := by simpa using I.ringCon.neg hx
Closure of Two-Sided Ideal Under Negation
Informal description
For any element $x$ in a two-sided ideal $I$ of a non-unital non-associative ring $R$, the negation $-x$ is also in $I$.
TwoSidedIdeal.instAddSubgroupClass instance
: AddSubgroupClass (TwoSidedIdeal R) R
Full source
instance : AddSubgroupClass (TwoSidedIdeal R) R where
  zero_mem := zero_mem
  add_mem := @add_mem _ _
  neg_mem := @neg_mem _ _
Two-Sided Ideals as Additive Subgroup Class
Informal description
For any non-unital non-associative ring $R$, the type of two-sided ideals of $R$ forms an additive subgroup class. This means that every two-sided ideal $I$ of $R$ is an additive subgroup of $R$, closed under addition and negation, and contains the zero element.
TwoSidedIdeal.sub_mem theorem
{x y} (hx : x ∈ I) (hy : y ∈ I) : x - y ∈ I
Full source
lemma sub_mem {x y} (hx : x ∈ I) (hy : y ∈ I) : x - y ∈ I := _root_.sub_mem hx hy
Closure of Two-Sided Ideal Under Subtraction
Informal description
For any elements $x$ and $y$ in a two-sided ideal $I$ of a non-unital non-associative ring $R$, the difference $x - y$ is also in $I$.
TwoSidedIdeal.mul_mem_left theorem
(x y) (hy : y ∈ I) : x * y ∈ I
Full source
lemma mul_mem_left (x y) (hy : y ∈ I) : x * y ∈ I := by
  simpa using I.ringCon.mul (I.ringCon.refl x) hy
Left Multiplication Preserves Ideal Membership
Informal description
For any elements $x, y$ in a non-unital non-associative ring $R$ and any two-sided ideal $I$ of $R$, if $y \in I$, then the product $x * y$ is also in $I$.
TwoSidedIdeal.mul_mem_right theorem
(x y) (hx : x ∈ I) : x * y ∈ I
Full source
lemma mul_mem_right (x y) (hx : x ∈ I) : x * y ∈ I := by
  simpa using I.ringCon.mul hx (I.ringCon.refl y)
Right Multiplication Preserves Ideal Membership
Informal description
For any elements $x, y$ in a non-unital non-associative ring $R$ and any two-sided ideal $I$ of $R$, if $x \in I$, then the product $x * y$ is also in $I$.
TwoSidedIdeal.nsmul_mem theorem
{x} (n : ℕ) (hx : x ∈ I) : n • x ∈ I
Full source
lemma nsmul_mem {x} (n : ) (hx : x ∈ I) : n • x ∈ I := _root_.nsmul_mem hx _
Natural number scalar multiplication preserves ideal membership
Informal description
For any element $x$ in a two-sided ideal $I$ of a non-unital non-associative ring $R$, and for any natural number $n$, the scalar multiple $n \cdot x$ is also in $I$.
TwoSidedIdeal.zsmul_mem theorem
{x} (n : ℤ) (hx : x ∈ I) : n • x ∈ I
Full source
lemma zsmul_mem {x} (n : ) (hx : x ∈ I) : n • x ∈ I := _root_.zsmul_mem hx _
Integer Scalar Multiplication Preserves Ideal Membership
Informal description
For any element $x$ in a non-unital non-associative ring $R$ and any two-sided ideal $I$ of $R$, if $x \in I$, then for any integer $n$, the scalar multiple $n \cdot x$ is also in $I$.
TwoSidedIdeal.mk' definition
(carrier : Set R) (zero_mem : 0 ∈ carrier) (add_mem : ∀ {x y}, x ∈ carrier → y ∈ carrier → x + y ∈ carrier) (neg_mem : ∀ {x}, x ∈ carrier → -x ∈ carrier) (mul_mem_left : ∀ {x y}, y ∈ carrier → x * y ∈ carrier) (mul_mem_right : ∀ {x y}, x ∈ carrier → x * y ∈ carrier) : TwoSidedIdeal R
Full source
/--
The "set-theoretic-way" of constructing a two-sided ideal by providing:
- the underlying set `S`;
- a proof that `0 ∈ S`;
- a proof that `x + y ∈ S` if `x ∈ S` and `y ∈ S`;
- a proof that `-x ∈ S` if `x ∈ S`;
- a proof that `x * y ∈ S` if `y ∈ S`;
- a proof that `x * y ∈ S` if `x ∈ S`.
-/
def mk' (carrier : Set R)
    (zero_mem : 0 ∈ carrier)
    (add_mem : ∀ {x y}, x ∈ carriery ∈ carrierx + y ∈ carrier)
    (neg_mem : ∀ {x}, x ∈ carrier-x ∈ carrier)
    (mul_mem_left : ∀ {x y}, y ∈ carrierx * y ∈ carrier)
    (mul_mem_right : ∀ {x y}, x ∈ carrierx * y ∈ carrier) : TwoSidedIdeal R where
  ringCon :=
    { r := fun x y ↦ x - y ∈ carrier
      iseqv :=
      { refl := fun x ↦ by simpa using zero_mem
        symm := fun h ↦ by simpa using neg_mem h
        trans := fun {x y z} h1 h2 ↦ by
          simpa only [show x - z = (x - y) + (y - z) by abel] using add_mem h1 h2 }
      mul' := fun {a b c d} (h1 : a - b ∈ carrier) (h2 : c - d ∈ carrier) ↦ show _ ∈ carrier by
        rw [show a * c - b * d = a * (c - d) + (a - b) * d by rw [mul_sub, sub_mul]; abel]
        exact add_mem (mul_mem_left h2) (mul_mem_right h1)
      add' := fun {a b c d} (h1 : a - b ∈ carrier) (h2 : c - d ∈ carrier) ↦ show _ ∈ carrier by
        rw [show a + c - (b + d) = (a - b) + (c - d) by abel]
        exact add_mem h1 h2 }
Construction of a two-sided ideal from a subset
Informal description
Given a non-unital non-associative ring \( R \), a two-sided ideal can be constructed from a subset \( S \subseteq R \) satisfying: 1. \( 0 \in S \); 2. \( x + y \in S \) for any \( x, y \in S \); 3. \( -x \in S \) for any \( x \in S \); 4. \( x \cdot y \in S \) for any \( x \in R \) and \( y \in S \); 5. \( x \cdot y \in S \) for any \( x \in S \) and \( y \in R \). The construction defines the ideal as the set of elements \( x \) such that \( x - y \in S \) for some \( y \), forming a congruence relation on \( R \).
TwoSidedIdeal.mem_mk' theorem
(carrier : Set R) (zero_mem add_mem neg_mem mul_mem_left mul_mem_right) (x : R) : x ∈ mk' carrier zero_mem add_mem neg_mem mul_mem_left mul_mem_right ↔ x ∈ carrier
Full source
@[simp]
lemma mem_mk' (carrier : Set R) (zero_mem add_mem neg_mem mul_mem_left mul_mem_right) (x : R) :
    x ∈ mk' carrier zero_mem add_mem neg_mem mul_mem_left mul_mem_rightx ∈ mk' carrier zero_mem add_mem neg_mem mul_mem_left mul_mem_right ↔ x ∈ carrier := by
  rw [mem_iff]
  simp [mk']
Membership Criterion for Constructed Two-Sided Ideal
Informal description
For a non-unital non-associative ring $R$, given a subset $S \subseteq R$ satisfying: 1. $0 \in S$, 2. $x + y \in S$ for all $x, y \in S$, 3. $-x \in S$ for all $x \in S$, 4. $x \cdot y \in S$ for all $x \in R$ and $y \in S$, 5. $x \cdot y \in S$ for all $x \in S$ and $y \in R$, an element $x \in R$ belongs to the two-sided ideal generated by $S$ if and only if $x \in S$.
TwoSidedIdeal.coe_mk' theorem
(carrier : Set R) (zero_mem add_mem neg_mem mul_mem_left mul_mem_right) : (mk' carrier zero_mem add_mem neg_mem mul_mem_left mul_mem_right : Set R) = carrier
Full source
@[simp]
lemma coe_mk' (carrier : Set R) (zero_mem add_mem neg_mem mul_mem_left mul_mem_right) :
    (mk' carrier zero_mem add_mem neg_mem mul_mem_left mul_mem_right : Set R) = carrier :=
  Set.ext <| mem_mk' carrier zero_mem add_mem neg_mem mul_mem_left mul_mem_right
Equality of Constructed Two-Sided Ideal with its Generating Set: $I(S) = S$
Informal description
For a non-unital non-associative ring $R$, given a subset $S \subseteq R$ satisfying: 1. $0 \in S$, 2. $x + y \in S$ for all $x, y \in S$, 3. $-x \in S$ for all $x \in S$, 4. $x \cdot y \in S$ for all $x \in R$ and $y \in S$, 5. $x \cdot y \in S$ for all $x \in S$ and $y \in R$, the underlying set of the two-sided ideal constructed from $S$ via `mk'` is equal to $S$ itself. That is, $(mk'\, S\, \text{zero\_mem}\, \text{add\_mem}\, \text{neg\_mem}\, \text{mul\_mem\_left}\, \text{mul\_mem\_right}) = S$.
TwoSidedIdeal.instSMulMemClass instance
: SMulMemClass (TwoSidedIdeal R) R R
Full source
instance : SMulMemClass (TwoSidedIdeal R) R R where
  smul_mem _ _ h := TwoSidedIdeal.mul_mem_left _ _ _ h
Two-sided Ideals are Closed under Left Multiplication
Informal description
For any non-unital non-associative ring $R$, the two-sided ideals of $R$ are closed under left multiplication by elements of $R$. That is, for any two-sided ideal $I$ and any elements $x \in R$ and $y \in I$, the product $x \cdot y$ belongs to $I$.
TwoSidedIdeal.instSMulMemClassMulOpposite instance
: SMulMemClass (TwoSidedIdeal R) Rᵐᵒᵖ R
Full source
instance : SMulMemClass (TwoSidedIdeal R) Rᵐᵒᵖ R where
  smul_mem _ _ h := TwoSidedIdeal.mul_mem_right _ _ _ h
Two-sided Ideals are Closed under Scalar Multiplication by Opposite Ring Elements
Informal description
For any non-unital non-associative ring $R$, a two-sided ideal $I$ of $R$ is closed under scalar multiplication by elements from the multiplicative opposite ring $R^\text{op}$. That is, for any $r \in R^\text{op}$ and $x \in I$, the product $r \cdot x$ is also in $I$.
TwoSidedIdeal.instAddSubtypeMem instance
: Add I
Full source
instance : Add I where add x y := ⟨x.1 + y.1, I.add_mem x.2 y.2⟩
Additive Structure on Two-sided Ideals
Informal description
For any two-sided ideal $I$ of a non-unital non-associative ring $R$, the subset $I$ inherits an additive structure from $R$, making it an additive subgroup.
TwoSidedIdeal.instZeroSubtypeMem instance
: Zero I
Full source
instance : Zero I where zero := ⟨0, I.zero_mem⟩
Zero Element in Two-sided Ideal
Informal description
For any two-sided ideal $I$ of a non-unital non-associative ring $R$, the subset $I$ contains the zero element $0$.
TwoSidedIdeal.instSMulNatSubtypeMem instance
: SMul ℕ I
Full source
instance : SMul  I where smul n x := ⟨n • x.1, I.nsmul_mem n x.2⟩
Natural Number Scalar Multiplication on Two-sided Ideals
Informal description
For any two-sided ideal $I$ of a non-unital non-associative ring $R$, the subset $I$ is equipped with a natural number scalar multiplication operation, where $n \cdot x$ is defined as repeated addition of $x$ for $n$ times.
TwoSidedIdeal.instNegSubtypeMem instance
: Neg I
Full source
instance : Neg I where neg x := ⟨-x.1, I.neg_mem x.2⟩
Negation Operation on Two-sided Ideals
Informal description
For any two-sided ideal $I$ of a non-unital non-associative ring $R$, the subset $I$ is equipped with a negation operation.
TwoSidedIdeal.instSubSubtypeMem instance
: Sub I
Full source
instance : Sub I where sub x y := ⟨x.1 - y.1, I.sub_mem x.2 y.2⟩
Subtraction Operation on Two-sided Ideals
Informal description
For any two-sided ideal $I$ of a non-unital non-associative ring $R$, the subset $I$ is equipped with a subtraction operation.
TwoSidedIdeal.instSMulIntSubtypeMem instance
: SMul ℤ I
Full source
instance : SMul  I where smul n x := ⟨n • x.1, I.zsmul_mem n x.2⟩
Integer Scalar Multiplication on Two-sided Ideals
Informal description
For any two-sided ideal $I$ of a non-unital non-associative ring $R$, there is a canonical scalar multiplication operation $\mathbb{Z} \times I \to I$ defined on $I$.
TwoSidedIdeal.addCommGroup instance
: AddCommGroup I
Full source
instance addCommGroup : AddCommGroup I :=
  Function.Injective.addCommGroup _ Subtype.coe_injective
    rfl (fun _ _ ↦ rfl) (fun _ ↦ rfl) (fun _ _ ↦ rfl) (fun _ _ ↦ rfl) (fun _ _ ↦ rfl)
Additive Commutative Group Structure on Two-sided Ideals
Informal description
For any two-sided ideal $I$ of a non-unital non-associative ring $R$, the subset $I$ forms an additive commutative group under the ring operations inherited from $R$.
TwoSidedIdeal.coeAddMonoidHom definition
: I →+ R
Full source
/-- The coercion into the ring as a `AddMonoidHom` -/
@[simps]
def coeAddMonoidHom : I →+ R where
  toFun := (↑)
  map_zero' := rfl
  map_add' _ _ := rfl
Canonical additive monoid homomorphism from a two-sided ideal to its ring
Informal description
The canonical additive monoid homomorphism from a two-sided ideal \( I \) of a non-unital non-associative ring \( R \) to \( R \) itself, which maps each element \( x \in I \) to its corresponding element in \( R \). This homomorphism preserves the additive structure, including the zero element and addition. More precisely, the homomorphism satisfies: 1. \( \text{coeAddMonoidHom}(0) = 0 \) (preservation of zero) 2. \( \text{coeAddMonoidHom}(x + y) = \text{coeAddMonoidHom}(x) + \text{coeAddMonoidHom}(y) \) for all \( x, y \in I \) (preservation of addition)
TwoSidedIdeal.op definition
(I : TwoSidedIdeal R) : TwoSidedIdeal Rᵐᵒᵖ
Full source
/-- If `I` is a two-sided ideal of `R`, then `{op x | x ∈ I}` is a two-sided ideal in `Rᵐᵒᵖ`. -/
@[simps]
def op (I : TwoSidedIdeal R) : TwoSidedIdeal Rᵐᵒᵖ where
  ringCon := I.ringCon.op
Two-sided ideal in the opposite ring
Informal description
Given a two-sided ideal \( I \) of a non-unital non-associative ring \( R \), the operation `TwoSidedIdeal.op` constructs a two-sided ideal in the opposite ring \( R^\text{op} \), consisting of all elements \( \text{op}(x) \) where \( x \in I \). Here, \( R^\text{op} \) is the ring with the same additive structure as \( R \) but with multiplication reversed.
TwoSidedIdeal.mem_op_iff theorem
{I : TwoSidedIdeal R} {x : Rᵐᵒᵖ} : x ∈ I.op ↔ x.unop ∈ I
Full source
@[simp]
lemma mem_op_iff {I : TwoSidedIdeal R} {x : Rᵐᵒᵖ} : x ∈ I.opx ∈ I.op ↔ x.unop ∈ I :=
  I.ringCon.comm'
Membership Criterion for Opposite Ideal: $x \in I^\text{op} \leftrightarrow x^\text{unop} \in I$
Informal description
For any two-sided ideal $I$ of a non-unital non-associative ring $R$ and any element $x$ in the opposite ring $R^\text{op}$, $x$ belongs to the opposite ideal $I^\text{op}$ if and only if the canonical projection of $x$ back to $R$ belongs to $I$. In symbols, for $x \in R^\text{op}$, \[ x \in I^\text{op} \leftrightarrow x^\text{unop} \in I. \]
TwoSidedIdeal.coe_op theorem
{I : TwoSidedIdeal R} : (I.op : Set Rᵐᵒᵖ) = MulOpposite.unop ⁻¹' I
Full source
@[simp, norm_cast]
lemma coe_op {I : TwoSidedIdeal R} : (I.op : Set Rᵐᵒᵖ) = MulOpposite.unopMulOpposite.unop ⁻¹' I :=
  Set.ext fun _ => mem_op_iff
Characterization of Opposite Ideal via Preimage: $I^\text{op} = \text{unop}^{-1}(I)$
Informal description
For any two-sided ideal $I$ of a non-unital non-associative ring $R$, the underlying set of the opposite ideal $I^\text{op}$ in the opposite ring $R^\text{op}$ is equal to the preimage of $I$ under the canonical projection $\text{unop} : R^\text{op} \to R$. In symbols, \[ I^\text{op} = \text{unop}^{-1}(I). \]
TwoSidedIdeal.unop definition
(I : TwoSidedIdeal Rᵐᵒᵖ) : TwoSidedIdeal R
Full source
/-- If `I` is a two-sided ideal of `Rᵐᵒᵖ`, then `{x.unop | x ∈ I}` is a two-sided ideal in `R`. -/
@[simps]
def unop (I : TwoSidedIdeal Rᵐᵒᵖ) : TwoSidedIdeal R where
  ringCon := I.ringCon.unop
Two-sided ideal in original ring from opposite ring
Informal description
Given a two-sided ideal $I$ of the opposite ring $R^\text{op}$, the function returns the two-sided ideal of $R$ consisting of all elements $x \in R$ such that $\text{op}(x) \in I$, where $\text{op} : R \to R^\text{op}$ is the canonical embedding.
TwoSidedIdeal.mem_unop_iff theorem
{I : TwoSidedIdeal Rᵐᵒᵖ} {x : R} : x ∈ I.unop ↔ MulOpposite.op x ∈ I
Full source
@[simp]
lemma mem_unop_iff {I : TwoSidedIdeal Rᵐᵒᵖ} {x : R} : x ∈ I.unopx ∈ I.unop ↔ MulOpposite.op x ∈ I :=
  I.ringCon.comm'
Membership Criterion for Two-sided Ideal via Opposite Ring
Informal description
For any two-sided ideal $I$ of the opposite ring $R^\text{op}$ and any element $x \in R$, $x$ belongs to the two-sided ideal $I.\text{unop}$ in $R$ if and only if the canonical embedding $\text{op}(x)$ belongs to $I$ in $R^\text{op}$.
TwoSidedIdeal.coe_unop theorem
{I : TwoSidedIdeal Rᵐᵒᵖ} : (I.unop : Set R) = MulOpposite.op ⁻¹' I
Full source
@[simp, norm_cast]
lemma coe_unop {I : TwoSidedIdeal Rᵐᵒᵖ} : (I.unop : Set R) = MulOpposite.opMulOpposite.op ⁻¹' I :=
  Set.ext fun _ => mem_unop_iff
Characterization of Unop Ideal via Preimage: $(I.\text{unop}) = \text{op}^{-1}(I)$
Informal description
For any two-sided ideal $I$ of the opposite ring $R^\text{op}$, the underlying set of the two-sided ideal $I.\text{unop}$ in $R$ is equal to the preimage of $I$ under the canonical embedding $\text{op} : R \to R^\text{op}$.
TwoSidedIdeal.opOrderIso definition
: TwoSidedIdeal R ≃o TwoSidedIdeal Rᵐᵒᵖ
Full source
/--
Two-sided-ideals of `A` and that of `Aᵒᵖ` corresponds bijectively to each other.
-/
@[simps]
def opOrderIso : TwoSidedIdealTwoSidedIdeal R ≃o TwoSidedIdeal Rᵐᵒᵖ where
  toFun := op
  invFun := unop
  left_inv _ := rfl
  right_inv _ := rfl
  map_rel_iff' {I' J'} := by simpa [ringCon_le_iff] using RingCon.opOrderIso.map_rel_iff
Order isomorphism between two-sided ideals and their opposites
Informal description
The order isomorphism between the lattice of two-sided ideals of a non-unital non-associative ring \( R \) and the lattice of two-sided ideals of its opposite ring \( R^\text{op} \). Specifically, it maps a two-sided ideal \( I \) of \( R \) to the two-sided ideal \( \text{op}(I) \) of \( R^\text{op} \), and vice versa via the inverse map \( \text{unop} \), preserving the order structure in both directions.