Documentation

Mathlib.Algebra.Module.Opposite

Module operations on Mᵐᵒᵖ #

This file contains definitions that build on top of the group action definitions in Mathlib.Algebra.GroupWithZero.Action.Opposite.

@[instance 910]

Like Semiring.toModule, but multiplies on the right.

Equations
instance MulOpposite.instModule (R : Type u) {M : Type v} [Semiring R] [AddCommMonoid M] [Module R M] :

MulOpposite.distribMulAction extends to a Module

Equations