Skip to content

Commit

Permalink
feat(group_theory/order_of_element): pow_eq_mod_card (#8354)
Browse files Browse the repository at this point in the history


Co-authored-by: Chris Hughes <33847686+ChrisHughes24@users.noreply.github.com>
  • Loading branch information
ChrisHughes24 and ChrisHughes24 committed Jul 20, 2021
1 parent 0f9b754 commit c05c15f
Showing 1 changed file with 10 additions and 0 deletions.
10 changes: 10 additions & 0 deletions src/group_theory/order_of_element.lean
Expand Up @@ -771,6 +771,16 @@ begin
exact pow_card_eq_one,
end

@[to_additive nsmul_eq_mod_card] lemma pow_eq_mod_card (n : ℕ) :
x ^ n = x ^ (n % fintype.card G) :=
by rw [pow_eq_mod_order_of, ←nat.mod_mod_of_dvd n order_of_dvd_card_univ,
← pow_eq_mod_order_of]

@[to_additive] lemma gpow_eq_mod_card (n : ℤ) :
x ^ n = x ^ (n % fintype.card G) :=
by by rw [gpow_eq_mod_order_of, ← int.mod_mod_of_dvd n (int.coe_nat_dvd.2 order_of_dvd_card_univ),
← gpow_eq_mod_order_of]

attribute [to_additive card_nsmul_eq_zero] pow_card_eq_one

/-- If `gcd(|G|,n)=1` then the `n`th power map is a bijection -/
Expand Down

0 comments on commit c05c15f

Please sign in to comment.