Skip to content

Commit

Permalink
chore(*): tweaks taken from gh-8889 (#10829)
Browse files Browse the repository at this point in the history
That PR is stale, but contained some trivial changes we should just take.
  • Loading branch information
eric-wieser committed Dec 15, 2021
1 parent 8218a78 commit 5a835b7
Show file tree
Hide file tree
Showing 2 changed files with 5 additions and 2 deletions.
1 change: 1 addition & 0 deletions src/analysis/complex/circle.lean
Expand Up @@ -102,6 +102,7 @@ subtype.ext $ by simp only [exp_map_circle_apply, submonoid.coe_mul, of_real_add

/-- The map `λ t, exp (t * I)` from `ℝ` to the unit circle in `ℂ`, considered as a homomorphism of
groups. -/
@[simps]
def exp_map_circle_hom : ℝ →+ (additive circle) :=
{ to_fun := additive.of_mul ∘ exp_map_circle,
map_zero' := exp_map_circle_zero,
Expand Down
6 changes: 4 additions & 2 deletions src/group_theory/quotient_group.lean
Expand Up @@ -124,10 +124,12 @@ lemma coe_inv (a : G) : ((a⁻¹ : G) : Q) = a⁻¹ := rfl
@[simp, to_additive quotient_add_group.coe_sub]
lemma coe_div (a b : G) : ((a / b : G) : Q) = a / b := by simp [div_eq_mul_inv]

@[simp] lemma coe_pow (a : G) (n : ℕ) : ((a ^ n : G) : Q) = a ^ n :=
@[simp, to_additive quotient_add_group.coe_nsmul]
lemma coe_pow (a : G) (n : ℕ) : ((a ^ n : G) : Q) = a ^ n :=
(mk' N).map_pow a n

@[simp] lemma coe_zpow (a : G) (n : ℤ) : ((a ^ n : G) : Q) = a ^ n :=
@[simp, to_additive quotient_add_group.coe_zsmul]
lemma coe_zpow (a : G) (n : ℤ) : ((a ^ n : G) : Q) = a ^ n :=
(mk' N).map_zpow a n

/-- A group homomorphism `φ : G →* H` with `N ⊆ ker(φ)` descends (i.e. `lift`s) to a
Expand Down

0 comments on commit 5a835b7

Please sign in to comment.