Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit a714245

Browse files
committed
feat(group_theory/order_of_element): order_of_dvd_iff_pow_eq_one (#2364)
1 parent 55814dc commit a714245

File tree

1 file changed

+3
-0
lines changed

1 file changed

+3
-0
lines changed

src/group_theory/order_of_element.lean

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -146,6 +146,9 @@ by_contradiction
146146
from nat.mod_lt _ (order_of_pos _))
147147
⟨nat.pos_of_ne_zero (mt nat.dvd_of_mod_eq_zero h₁), by rwa ← pow_eq_mod_order_of⟩)
148148

149+
lemma order_of_dvd_iff_pow_eq_one {n : ℕ} : order_of a ∣ n ↔ a ^ n = 1 :=
150+
⟨λ h, by rw [pow_eq_mod_order_of, nat.mod_eq_zero_of_dvd h, pow_zero], order_of_dvd_of_pow_eq_one⟩
151+
149152
lemma order_of_le_of_pow_eq_one {n : ℕ} (hn : 0 < n) (h : a ^ n = 1) : order_of a ≤ n :=
150153
nat.find_min' (exists_pow_eq_one a) ⟨hn, h⟩
151154

0 commit comments

Comments
 (0)