Skip to content

Commit 09b44c1

Browse files
committed
feat(GroupTheory/GroupAction/Group): invOf smul lemmas (#9972)
Give `smul` versions of some existing `mul` lemmas: - `invOf_smul_smul` - smul_invOf_smul (c.f. mul_invOf_self_assoc) - `invOf_smul_eq_iff` (c.f. `invOf_mul_eq_iff_eq_mul_left`) (required for #7569) - `smul_eq_iff_eq_invOf_smul` (c.f `mul_left_eq_iff_eq_invOf_mul`) Co-authored-by: Christopher Hoskin <christopher.hoskin@overleaf.com> Co-authored-by: Christopher Hoskin <mans0954@users.noreply.github.com>
1 parent e4e10f9 commit 09b44c1

File tree

1 file changed

+23
-0
lines changed

1 file changed

+23
-0
lines changed

Mathlib/GroupTheory/GroupAction/Group.lean

Lines changed: 23 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Chris Hughes
55
-/
66
import Mathlib.Algebra.Group.Aut
7+
import Mathlib.Algebra.Invertible.Basic
78
import Mathlib.GroupTheory.GroupAction.Units
89

910
#align_import group_theory.group_action.group from "leanprover-community/mathlib"@"3b52265189f3fb43aa631edffce5d060fafaf82f"
@@ -178,6 +179,28 @@ theorem smul_eq_iff_eq_inv_smul (g : α) {x y : β} : g • x = y ↔ x = g⁻¹
178179

179180
end Group
180181

182+
section Monoid
183+
184+
variable [Monoid α] [MulAction α β]
185+
186+
variable (c : α) (x y : β) [Invertible c]
187+
188+
@[simp]
189+
theorem invOf_smul_smul : ⅟c • c • x = x := inv_smul_smul (unitOfInvertible c) _
190+
191+
@[simp]
192+
theorem smul_invOf_smul : c • (⅟ c • x) = x := smul_inv_smul (unitOfInvertible c) _
193+
194+
variable {c x y}
195+
196+
theorem invOf_smul_eq_iff : ⅟c • x = y ↔ x = c • y :=
197+
inv_smul_eq_iff (a := unitOfInvertible c)
198+
199+
theorem smul_eq_iff_eq_invOf_smul : c • x = y ↔ x = ⅟c • y :=
200+
smul_eq_iff_eq_inv_smul (g := unitOfInvertible c)
201+
202+
end Monoid
203+
181204
/-- `Monoid.toMulAction` is faithful on nontrivial cancellative monoids with zero. -/
182205
instance CancelMonoidWithZero.faithfulSMul [CancelMonoidWithZero α] [Nontrivial α] :
183206
FaithfulSMul α α :=

0 commit comments

Comments
 (0)