theorem
Commute.ofNat_left
{α : Type u_1}
[NonAssocSemiring α]
(n : ℕ)
[n.AtLeastTwo]
(x : α)
 :
Commute (OfNat.ofNat n) x
theorem
Commute.ofNat_right
{α : Type u_1}
[NonAssocSemiring α]
(x : α)
(n : ℕ)
[n.AtLeastTwo]
 :
Commute x (OfNat.ofNat n)
@[simp]
theorem
SemiconjBy.natCast_mul_right
{α : Type u_1}
[Semiring α]
{a : α}
{x : α}
{y : α}
(h : SemiconjBy a x y)
(n : ℕ)
 :
SemiconjBy a (↑n * x) (↑n * y)
@[simp]
theorem
SemiconjBy.natCast_mul_left
{α : Type u_1}
[Semiring α]
{a : α}
{x : α}
{y : α}
(h : SemiconjBy a x y)
(n : ℕ)
 :
SemiconjBy (↑n * a) x y
@[simp]
theorem
SemiconjBy.natCast_mul_natCast_mul
{α : Type u_1}
[Semiring α]
{a : α}
{x : α}
{y : α}
(h : SemiconjBy a x y)
(m : ℕ)
(n : ℕ)
 :
SemiconjBy (↑m * a) (↑n * x) (↑n * y)
@[deprecated Commute.natCast_mul_right]
theorem
Commute.cast_nat_mul_right
{α : Type u_1}
[Semiring α]
{a : α}
{b : α}
(h : Commute a b)
(n : ℕ)
 :
Alias of Commute.natCast_mul_right.
@[deprecated Commute.natCast_mul_left]
theorem
Commute.cast_nat_mul_left
{α : Type u_1}
[Semiring α]
{a : α}
{b : α}
(h : Commute a b)
(n : ℕ)
 :
Alias of Commute.natCast_mul_left.
@[deprecated Commute.self_natCast_mul]
Alias of Commute.self_natCast_mul.
@[deprecated Commute.natCast_mul_self]
Alias of Commute.natCast_mul_self.
@[deprecated Commute.self_natCast_mul_natCast_mul]
theorem
Commute.self_cast_nat_mul_cast_nat_mul
{α : Type u_1}
[Semiring α]
(a : α)
(m : ℕ)
(n : ℕ)
 :
Alias of Commute.self_natCast_mul_natCast_mul.