theorem
left_inverse_neg
(G : Type u_1)
[add_group G] :
function.left_inverse (λ (a : G), -a) (λ (a : G), -a)
theorem
left_inverse_inv
(G : Type u_1)
[group G] :
function.left_inverse (λ (a : G), a⁻¹) (λ (a : G), a⁻¹)
theorem
mul_right_surjective
{G : Type u}
[group G]
(a : G) :
function.surjective (λ (x : G), x * a)
theorem
add_right_surjective
{G : Type u}
[add_group G]
(a : G) :
function.surjective (λ (x : G), x + a)
theorem
left_inverse_sub_add_left
{G : Type u}
[add_group G]
(c : G) :
function.left_inverse (λ (x : G), x - c) (λ (x : G), x + c)
theorem
left_inverse_add_left_sub
{G : Type u}
[add_group G]
(c : G) :
function.left_inverse (λ (x : G), x + c) (λ (x : G), x - c)
theorem
left_inverse_add_right_neg_add
{G : Type u}
[add_group G]
(c : G) :
function.left_inverse (λ (x : G), c + x) (λ (x : G), -c + x)
theorem
left_inverse_neg_add_add_right
{G : Type u}
[add_group G]
(c : G) :
function.left_inverse (λ (x : G), -c + x) (λ (x : G), c + x)
@[simp]
@[simp]
@[simp]