Congruences on the opposite of a group #
This file defines the order isomorphism between the congruences on a group G
and the congruences
on the opposite group Gᵒᵖ
.
If c
is an additive congruence on Mᵃᵒᵖ
, then (a, b) ↦ c bᵒᵖ aᵒᵖ
is an additive
congruence on M
Equations
- c.unop = { r := fun (a b : M) => c (AddOpposite.op b) (AddOpposite.op a), iseqv := ⋯, add' := ⋯ }
Instances For
The additive congruences on M
bijects to the additive congruences
on Mᵃᵒᵖ
Equations
- AddCon.orderIsoOp = { toFun := AddCon.op, invFun := AddCon.unop, left_inv := ⋯, right_inv := ⋯, map_rel_iff' := ⋯ }
Instances For
@[simp]
@[simp]
@[simp]