Skip to content

Commit 2d2ad99

Browse files
committed
1 parent 598f6c1 commit 2d2ad99

File tree

2 files changed

+11
-2
lines changed

2 files changed

+11
-2
lines changed

Mathlib/Algebra/GroupPower/Order.lean

Lines changed: 6 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Jeremy Avigad, Robert Y. Lewis
55
66
! This file was ported from Lean 3 source module algebra.group_power.order
7-
! leanprover-community/mathlib commit dd4c2044a9dee231309637e7fd4e61aea1506e33
7+
! leanprover-community/mathlib commit 00f91228655eecdcd3ac97a7fd8dbcb139fe990a
88
! Please do not edit these lines, except to modify the commit id
99
! if you have ported upstream changes.
1010
-/
@@ -634,6 +634,11 @@ theorem pow_abs (a : R) (n : ℕ) : |a| ^ n = |a ^ n| :=
634634
theorem abs_neg_one_pow (n : ℕ) : |(-1 : R) ^ n| = 1 := by rw [← pow_abs, abs_neg, abs_one, one_pow]
635635
#align abs_neg_one_pow abs_neg_one_pow
636636

637+
theorem abs_pow_eq_one (a : R) {n : ℕ} (h : 0 < n) : |a ^ n| = 1 ↔ |a| = 1 := by
638+
convert pow_left_inj (abs_nonneg a) zero_le_one h
639+
exacts [(pow_abs _ _).symm, (one_pow _).symm]
640+
#align abs_pow_eq_one abs_pow_eq_one
641+
637642
section
638643
set_option linter.deprecated false
639644

Mathlib/Algebra/Ring/Equiv.lean

Lines changed: 5 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5,7 +5,7 @@ Authors: Johannes Hölzl, Callum Sutton, Yury Kudryashov
55
Ported by: Anatole Dedecker
66
77
! This file was ported from Lean 3 source module algebra.ring.equiv
8-
! leanprover-community/mathlib commit a59dad53320b73ef180174aae867addd707ef00e
8+
! leanprover-community/mathlib commit 00f91228655eecdcd3ac97a7fd8dbcb139fe990a
99
! Please do not edit these lines, except to modify the commit id
1010
! if you have ported upstream changes.
1111
-/
@@ -583,6 +583,10 @@ theorem map_neg_one : f (-1) = -1 :=
583583
f.map_one ▸ f.map_neg 1
584584
#align ring_equiv.map_neg_one RingEquiv.map_neg_one
585585

586+
theorem map_eq_neg_one_iff {x : R} : f x = -1 ↔ x = -1 := by
587+
rw [← neg_eq_iff_eq_neg, ← neg_eq_iff_eq_neg, ← map_neg, RingEquiv.map_eq_one_iff]
588+
#align ring_equiv.map_eq_neg_one_iff RingEquiv.map_eq_neg_one_iff
589+
586590
end Ring
587591

588592
section NonUnitalSemiringHom

0 commit comments

Comments
 (0)