Semirings and rings #
This file gives lemmas about semirings, rings and domains.
This is analogous to Algebra.Group.Basic,
the difference being that the former is about + and * separately, while
the present file is about their interaction.
For the definitions of semirings and rings see Algebra.Ring.Defs.
Left multiplication by an element of a type with distributive multiplication is an AddHom.
Equations
- AddHom.mulLeft r = { toFun := fun (x : R) => r * x, map_add' := ⋯ }
Instances For
Left multiplication by an element of a type with distributive multiplication is an AddHom.
Equations
- AddHom.mulRight r = { toFun := fun (a : R) => a * r, map_add' := ⋯ }
Instances For
Left multiplication by an element of a (semi)ring is an AddMonoidHom
Equations
- AddMonoidHom.mulLeft r = { toFun := fun (x : R) => r * x, map_zero' := ⋯, map_add' := ⋯ }
Instances For
Right multiplication by an element of a (semi)ring is an AddMonoidHom
Equations
- AddMonoidHom.mulRight r = { toFun := fun (a : R) => a * r, map_zero' := ⋯, map_add' := ⋯ }
Instances For
Equations
- instHasDistribNeg = HasDistribNeg.mk ⋯ ⋯
Vieta's formula for a quadratic equation, relating the coefficients of the polynomial with
its roots. This particular version states that if we have a root x of a monic quadratic
polynomial, then there is another root y such that x + y is negative the a_1 coefficient
and x * y is the a_0 coefficient.
Equations
- ⋯ = ⋯
In a ring, IsCancelMulZero and NoZeroDivisors are equivalent.
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯