Skip to content

Commit

Permalink
feat(group_theory/subgroup/basic): Cyclic subgroups are commutative (#…
Browse files Browse the repository at this point in the history
…13663)

This PR adds an instance stating that the cyclic subgroups `zpowers g` are commutative.
  • Loading branch information
tb65536 committed Apr 25, 2022
1 parent b0fe3cd commit ef3769d
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions src/group_theory/subgroup/basic.lean
Expand Up @@ -2648,6 +2648,14 @@ begin
exact of_mul_image_zpowers_eq_zmultiples_of_mul,
end

namespace subgroup

@[to_additive] instance zpowers_is_commutative (g : G) : (zpowers g).is_commutative :=
⟨⟨λ ⟨_, _, h₁⟩ ⟨_, _, h₂⟩, by rw [subtype.ext_iff, coe_mul, coe_mul,
subtype.coe_mk, subtype.coe_mk, ←h₁, ←h₂, zpow_mul_comm]⟩⟩

end subgroup

namespace monoid_hom

variables {G' : Type*} [group G']
Expand Down

0 comments on commit ef3769d

Please sign in to comment.