Skip to content

Commit a48a515

Browse files
committed
chore: fix names in algebra/group (#580)
I might have missed a lemma or two, but I think that the folder is now good.
1 parent fa0fc4e commit a48a515

File tree

2 files changed

+20
-7
lines changed

2 files changed

+20
-7
lines changed

Mathlib/Algebra/Group/Basic.lean

Lines changed: 18 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -176,12 +176,16 @@ theorem inv_comp_inv : Inv.inv ∘ Inv.inv = @id G :=
176176
inv_involutive.comp_self
177177

178178
@[to_additive]
179-
theorem left_inverse_inv : LeftInverse (fun a : G => a⁻¹) fun a => a⁻¹ :=
179+
theorem leftInverse_inv : LeftInverse (fun a : G => a⁻¹) fun a => a⁻¹ :=
180180
inv_inv
181+
#align left_inverse_inv leftInverse_inv
182+
#align left_inverse_neg leftInverse_neg
181183

182184
@[to_additive]
183-
theorem right_inverse_inv : LeftInverse (fun a : G => a⁻¹) fun a => a⁻¹ :=
185+
theorem rightInverse_inv : LeftInverse (fun a : G => a⁻¹) fun a => a⁻¹ :=
184186
inv_inv
187+
#align right_inverse_inv rightInverse_inv
188+
#align right_inverse_neg rightInverse_neg
185189

186190
end HasInvolutiveInv
187191

@@ -554,22 +558,30 @@ theorem eq_iff_eq_of_div_eq_div (H : a / b = c / d) : a = b ↔ c = d :=
554558
by rw [← div_eq_one, H, div_eq_one]
555559

556560
@[to_additive]
557-
theorem left_inverse_div_mul_left (c : G) : Function.LeftInverse (fun x => x / c) fun x => x * c :=
561+
theorem leftInverse_div_mul_left (c : G) : Function.LeftInverse (fun x => x / c) fun x => x * c :=
558562
fun x => mul_div_cancel'' x c
563+
#align left_inverse_div_mul_left leftInverse_div_mul_left
564+
#align left_inverse_sub_add_left leftInverse_sub_add_left
559565

560566
@[to_additive]
561-
theorem left_inverse_mul_left_div (c : G) : Function.LeftInverse (fun x => x * c) fun x => x / c :=
567+
theorem leftInverse_mul_left_div (c : G) : Function.LeftInverse (fun x => x * c) fun x => x / c :=
562568
fun x => div_mul_cancel' x c
569+
#align left_inverse_mul_left_div leftInverse_mul_left_div
570+
#align left_inverse_add_left_sub leftInverse_add_left_sub
563571

564572
@[to_additive]
565-
theorem left_inverse_mul_right_inv_mul (c : G) :
573+
theorem leftInverse_mul_right_inv_mul (c : G) :
566574
Function.LeftInverse (fun x => c * x) fun x => c⁻¹ * x :=
567575
fun x => mul_inv_cancel_left c x
576+
#align left_inverse_mul_right_inv_mul leftInverse_mul_right_inv_mul
577+
#align left_inverse_add_right_neg_add leftInverse_add_right_neg_add
568578

569579
@[to_additive]
570-
theorem left_inverse_inv_mul_mul_right (c : G) :
580+
theorem leftInverse_inv_mul_mul_right (c : G) :
571581
Function.LeftInverse (fun x => c⁻¹ * x) fun x => c * x :=
572582
fun x => inv_mul_cancel_left c x
583+
#align left_inverse_inv_mul_mul_right leftInverse_inv_mul_mul_right
584+
#align left_inverse_neg_add_add_right leftInverse_neg_add_add_right
573585

574586
-- TODO @[to_additive]
575587
theorem exists_npow_eq_one_of_zpow_eq_one {n : ℤ} (hn : n ≠ 0) {x : G} (h : x ^ n = 1) :

Mathlib/Algebra/Group/Commute.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -57,8 +57,9 @@ protected theorem symm {a b : S} (h : Commute a b) : Commute b a :=
5757
Eq.symm h
5858

5959
@[to_additive]
60-
protected theorem semiconj_by {a b : S} (h : Commute a b) : SemiconjBy a b b :=
60+
protected theorem semiconjBy {a b : S} (h : Commute a b) : SemiconjBy a b b :=
6161
h
62+
#align commute.semiconj_by Commute.semiconjBy
6263

6364
@[to_additive]
6465
protected theorem symm_iff {a b : S} : Commute a b ↔ Commute b a :=

0 commit comments

Comments
 (0)