Skip to content

Commit

Permalink
feat(ring_theory/roots_of_unity): coe_injective (#11793)
Browse files Browse the repository at this point in the history
from flt-regular
  • Loading branch information
ericrbg committed Feb 3, 2022
1 parent 934f182 commit 50ee3d5
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions src/ring_theory/roots_of_unity.lean
Expand Up @@ -82,6 +82,9 @@ def roots_of_unity (k : ℕ+) (M : Type*) [comm_monoid M] : subgroup Mˣ :=
@[simp] lemma mem_roots_of_unity (k : ℕ+) (ζ : Mˣ) :
ζ ∈ roots_of_unity k M ↔ ζ ^ (k : ℕ) = 1 := iff.rfl

lemma roots_of_unity.coe_injective {n : ℕ+} : function.injective (coe : (roots_of_unity n M) → M) :=
units.ext.comp (λ x y, subtype.ext)

/-- Make an element of `roots_of_unity` from a member of the base ring, and a proof that it has
a positive power equal to one. -/
@[simps coe_coe] def roots_of_unity.mk_of_pow_eq (ζ : M) {n : ℕ+} (h : ζ ^ (n : ℕ) = 1) :
Expand Down

0 comments on commit 50ee3d5

Please sign in to comment.