Skip to content

Commit 487ae74

Browse files
pecherskywinstonyinkim-emj-loreauxRuben-VandeVelde
committedDec 2, 2022
feat: port Algebra.Hom.Group (#659)
mathlib3 SHA: 8c53048add6ffacdda0b36c4917bfe37e209b0ba - [x] depends on #563 - [x] depends on leanprover-community/mathlib3#17733 - [x] depends on leanprover/lean4#1901 - [x] depends on leanprover/lean4#1907 Co-authored-by: Winston Yin <winstonyin@gmail.com> Co-authored-by: Scott Morrison <scott.morrison@gmail.com> Co-authored-by: Jireh Loreaux <loreaujy@gmail.com> Co-authored-by: Ruben Van de Velde <65514131+Ruben-VandeVelde@users.noreply.github.com>
1 parent 5658b22 commit 487ae74

File tree

5 files changed

+1615
-3
lines changed

5 files changed

+1615
-3
lines changed
 

Diff for: ‎Mathlib.lean

+1
Original file line numberDiff line numberDiff line change
@@ -21,6 +21,7 @@ import Mathlib.Algebra.GroupWithZero.Semiconj
2121
import Mathlib.Algebra.GroupWithZero.Units.Basic
2222
import Mathlib.Algebra.HierarchyDesign
2323
import Mathlib.Algebra.Hom.Embedding
24+
import Mathlib.Algebra.Hom.Group
2425
import Mathlib.Algebra.Homology.ComplexShape
2526
import Mathlib.Algebra.NeZero
2627
import Mathlib.Algebra.Opposites

Diff for: ‎Mathlib/Algebra/Group/Defs.lean

+7-1
Original file line numberDiff line numberDiff line change
@@ -783,10 +783,16 @@ theorem zpow_ofNat (a : G) : ∀ n : ℕ, a ^ (n : ℤ) = a ^ n
783783
_ = a * a ^ n := congr_arg ((· * ·) a) (zpow_ofNat a n)
784784
_ = a ^ (n + 1) := (pow_succ _ _).symm
785785

786-
@[simp, to_additive]
786+
@[simp]
787787
theorem zpow_negSucc (a : G) (n : ℕ) : a ^ (Int.negSucc n) = (a ^ (n + 1))⁻¹ := by
788788
rw [← zpow_ofNat]
789789
exact DivInvMonoid.zpow_neg' n a
790+
@[simp]
791+
theorem negSucc_zsmul {G} [SubNegMonoid G] (a : G) (n : ℕ) :
792+
Int.negSucc n • a = -((n + 1) • a) := by
793+
rw [← ofNat_zsmul]
794+
exact SubNegMonoid.zsmul_neg' n a
795+
attribute [to_additive negSucc_zsmul] zpow_negSucc
790796

791797
/-- Dividing by an element is the same as multiplying by its inverse.
792798

Diff for: ‎Mathlib/Algebra/Hom/Group.lean

+1,605
Large diffs are not rendered by default.

Diff for: ‎Mathlib/Logic/Nonempty.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -21,7 +21,7 @@ This file proves a few extra facts about `Nonempty`, which is defined in core Le
2121

2222
variable {γ : α → Type _}
2323

24-
instance (priority := 20) Zero.Nonempty [Zero α] : Nonempty α :=
24+
instance (priority := 20) Zero.nonempty [Zero α] : Nonempty α :=
2525
0
2626

2727
instance (priority := 20) One.nonempty [One α] : Nonempty α :=

Diff for: ‎lean-toolchain

+1-1
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:nightly-2022-12-02
1+
semorrison/lean4:fix-1907

0 commit comments

Comments
 (0)
Please sign in to comment.