Skip to content

Commit

Permalink
feat(group_theory/subgroup/basic): Alternate version of `mem_normaliz…
Browse files Browse the repository at this point in the history
…er_iff` (#12814)

This PR adds an alternate version of `mem_normalizer_iff`, in terms of commuting rather than conjugation.
  • Loading branch information
tb65536 committed Mar 19, 2022
1 parent 52b9b36 commit 3ba1c02
Showing 1 changed file with 9 additions and 0 deletions.
9 changes: 9 additions & 0 deletions src/group_theory/subgroup/basic.lean
Expand Up @@ -1507,6 +1507,15 @@ variable {H}
@[to_additive] lemma mem_normalizer_iff {g : G} :
g ∈ normalizer H ↔ ∀ n, n ∈ H ↔ g * n * g⁻¹ ∈ H := iff.rfl

@[to_additive] lemma mem_normalizer_iff' {g : G} : g ∈ normalizer H ↔ ∀ n, n * g ∈ H ↔ g * n ∈ H :=
begin
refine ⟨λ h n, _, λ h n, _⟩,
{ specialize h (n * g),
rwa [mul_assoc, mul_inv_cancel_right] at h },
{ specialize h (n * g⁻¹),
rwa [inv_mul_cancel_right, ←mul_assoc] at h },
end

@[to_additive] lemma le_normalizer : H ≤ normalizer H :=
λ x xH n, by rw [H.mul_mem_cancel_right (H.inv_mem xH), H.mul_mem_cancel_left xH]

Expand Down

0 comments on commit 3ba1c02

Please sign in to comment.