Scalar multiplication on ℝ≥0∞
. #
This file defines basic scalar actions on extended nonnegative reals, showing that
MulAction
s, DistribMulAction
s, Module
s and Algebra
s restrict from ℝ≥0∞
to ℝ≥0
.
instance
ENNReal.instIsScalarTowerNNReal
{M : Type u_1}
{N : Type u_2}
[MulAction ENNReal M]
[MulAction ENNReal N]
[SMul M N]
[IsScalarTower ENNReal M N]
:
IsScalarTower NNReal M N
instance
ENNReal.smulCommClass_left
{M : Type u_1}
{N : Type u_2}
[MulAction ENNReal N]
[SMul M N]
[SMulCommClass ENNReal M N]
:
SMulCommClass NNReal M N
instance
ENNReal.smulCommClass_right
{M : Type u_1}
{N : Type u_2}
[MulAction ENNReal N]
[SMul M N]
[SMulCommClass M ENNReal N]
:
SMulCommClass M NNReal N
noncomputable instance
ENNReal.instDistribMulActionNNReal
{M : Type u_1}
[AddMonoid M]
[DistribMulAction ENNReal M]
:
A DistribMulAction
over ℝ≥0∞
restricts to a DistribMulAction
over ℝ≥0
.
noncomputable instance
ENNReal.instModuleNNReal
{M : Type u_1}
[AddCommMonoid M]
[Module ENNReal M]
:
theorem
ENNReal.smul_top
{R : Type u_1}
[Zero R]
[SMulWithZero R ENNReal]
[IsScalarTower R ENNReal ENNReal]
[NoZeroSMulDivisors R ENNReal]
[DecidableEq R]
(c : R)
: