Documentation

Mathlib.RingTheory.Congruence.Opposite

Congruences on the opposite ring #

This file defines the order isomorphism between the congruences on a ring R and the congruences on the opposite ring Rᵐᵒᵖ.

def RingCon.op {R : Type u_1} [Add R] [Mul R] (c : RingCon R) :

If c is a RingCon R, then (a, b) ↦ c b.unop a.unop is a RingCon Rᵐᵒᵖ.

Equations
Instances For
    theorem RingCon.op_iff {R : Type u_1} [Add R] [Mul R] {c : RingCon R} {x y : Rᵐᵒᵖ} :
    def RingCon.unop {R : Type u_1} [Add R] [Mul R] (c : RingCon Rᵐᵒᵖ) :

    If c is a RingCon Rᵐᵒᵖ, then (a, b) ↦ c b.op a.op is a RingCon R.

    Equations
    Instances For
      theorem RingCon.unop_iff {R : Type u_1} [Add R] [Mul R] {c : RingCon Rᵐᵒᵖ} {x y : R} :

      The congruences of a ring R biject to the congruences of the opposite ring Rᵐᵒᵖ.

      Equations
      Instances For
        @[simp]
        theorem RingCon.opOrderIso_apply {R : Type u_1} [Add R] [Mul R] (c : RingCon R) :