Skip to content
This repository has been archived by the owner on Jul 24, 2024. It is now read-only.

Commit

Permalink
feat(group_theory/subgroup/pointwise): Basic lemmas (#16856)
Browse files Browse the repository at this point in the history
This PR adds some basic lemmas `smul_bot`, `smul_inf`, and `smul_normal` (a restatement of `normal.conj_act` in terms of `mul_aut.conj`).
  • Loading branch information
tb65536 committed Oct 11, 2022
1 parent 03eaefc commit 21926ff
Showing 1 changed file with 9 additions and 0 deletions.
9 changes: 9 additions & 0 deletions src/group_theory/subgroup/pointwise.lean
Original file line number Diff line number Diff line change
Expand Up @@ -60,6 +60,9 @@ lemma mem_smul_pointwise_iff_exists (m : G) (a : α) (S : subgroup G) :
m ∈ a • S ↔ ∃ (s : G), s ∈ S ∧ a • s = m :=
(set.mem_smul_set : m ∈ a • (S : set G) ↔ _)

@[simp] lemma smul_bot (a : α) : a • (⊥ : subgroup G) = ⊥ :=
by simp [set_like.ext_iff, mem_smul_pointwise_iff_exists, eq_comm]

instance pointwise_central_scalar [mul_distrib_mul_action αᵐᵒᵖ G] [is_central_scalar α G] :
is_central_scalar α (subgroup G) :=
⟨λ a S, congr_arg (λ f, S.map f) $ monoid_hom.ext $ by exact op_smul_eq_smul _⟩
Expand Down Expand Up @@ -109,6 +112,9 @@ set_smul_subset_iff
lemma subset_pointwise_smul_iff {a : α} {S T : subgroup G} : S ≤ a • T ↔ a⁻¹ • S ≤ T :=
subset_set_smul_iff

@[simp] lemma smul_inf (a : α) (S T : subgroup G) : a • (S ⊓ T) = a • S ⊓ a • T :=
by simp [set_like.ext_iff, mem_pointwise_smul_iff_inv_smul_mem]

/-- Applying a `mul_distrib_mul_action` results in an isomorphic subgroup -/
@[simps] def equiv_smul (a : α) (H : subgroup G) : H ≃* (a • H : subgroup G) :=
(mul_distrib_mul_action.to_mul_equiv G a).subgroup_map H
Expand Down Expand Up @@ -152,6 +158,9 @@ begin
exact h}
end

@[simp] lemma smul_normal (g : G) (H : subgroup G) [h : normal H] : mul_aut.conj g • H = H :=
h.conj_act g

end group

section group_with_zero
Expand Down

0 comments on commit 21926ff

Please sign in to comment.