Documentation
Mathlib
.
Algebra
.
Ring
.
Action
.
Rat
Search
return to top
source
Imports
Init
Mathlib.Algebra.Field.Defs
Mathlib.Algebra.GroupWithZero.Action.Defs
Imported by
NNRat
.
instDistribSMul
NNRat
.
instIsScalarTowerRight
Rat
.
instDistribSMul
Rat
.
instIsScalarTowerRight
Actions by nonnegative rational numbers
#
Scalar multiplication
#
source
@[instance 100]
instance
NNRat
.
instDistribSMul
{
R
:
Type
u_1}
[
DivisionSemiring
R
]
:
DistribSMul
ℚ≥0
R
Equations
NNRat.instDistribSMul
=
DistribSMul.mk
⋯
source
instance
NNRat
.
instIsScalarTowerRight
{
R
:
Type
u_1}
[
DivisionSemiring
R
]
:
IsScalarTower
ℚ≥0
R
R
source
@[instance 100]
instance
Rat
.
instDistribSMul
{
R
:
Type
u_1}
[
DivisionRing
R
]
:
DistribSMul
ℚ
R
Equations
Rat.instDistribSMul
=
DistribSMul.mk
⋯
source
instance
Rat
.
instIsScalarTowerRight
{
R
:
Type
u_1}
[
DivisionRing
R
]
:
IsScalarTower
ℚ
R
R