The embedding of a cancellative semigroup into itself by multiplication by a fixed element. #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
The embedding of a left cancellative additive semigroup into itself by left translation by a fixed element.
The embedding of a left cancellative semigroup into itself by left multiplication by a fixed element.
@[simp]
theorem
add_left_embedding_apply
{G : Type u_1}
[add_left_cancel_semigroup G]
(g h : G) :
⇑(add_left_embedding g) h = g + h
@[simp]
theorem
mul_left_embedding_apply
{G : Type u_1}
[left_cancel_semigroup G]
(g h : G) :
⇑(mul_left_embedding g) h = g * h
@[simp]
theorem
add_right_embedding_apply
{G : Type u_1}
[add_right_cancel_semigroup G]
(g h : G) :
⇑(add_right_embedding g) h = h + g
The embedding of a right cancellative semigroup into itself by right multiplication by a fixed element.
The embedding of a right cancellative additive semigroup into itself by right translation by a fixed element.
@[simp]
theorem
mul_right_embedding_apply
{G : Type u_1}
[right_cancel_semigroup G]
(g h : G) :
⇑(mul_right_embedding g) h = h * g
theorem
add_left_embedding_eq_add_right_embedding
{G : Type u_1}
[add_cancel_comm_monoid G]
(g : G) :