Skip to content

Commit

Permalink
feat(algebra/group_power/order): Add sq_zero_iff (#13670)
Browse files Browse the repository at this point in the history
Tiny lemma that seems to be missing.

Should this be a simp lemma?

Co-authored-by: Yury G. Kudryashov <urkud@urkud.name>
  • Loading branch information
Smaug123 and urkud committed Apr 25, 2022
1 parent e2f5696 commit 4481a56
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions src/algebra/group_power/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -330,6 +330,9 @@ lemma pow_ne_zero_iff [monoid_with_zero R] [no_zero_divisors R] {a : R} {n : ℕ
{a : R} (n : ℕ) (h : a ≠ 0) : a ^ n ≠ 0 :=
mt pow_eq_zero h

theorem sq_eq_zero_iff [monoid_with_zero R] [no_zero_divisors R] {a : R} : a ^ 2 = 0 ↔ a = 0 :=
pow_eq_zero_iff two_pos

lemma pow_dvd_pow_iff [cancel_comm_monoid_with_zero R]
{x : R} {n m : ℕ} (h0 : x ≠ 0) (h1 : ¬ is_unit x) :
x ^ n ∣ x ^ m ↔ n ≤ m :=
Expand Down

0 comments on commit 4481a56

Please sign in to comment.