Skip to content

Commit

Permalink
feat(group_theory/subgroup/basic): golf proof of instance normal_inf_…
Browse files Browse the repository at this point in the history
…normal (#16620)

Removed some `rw` from the proof of the instance `normal_inf_normal`.
  • Loading branch information
faenuccio committed Sep 26, 2022
1 parent ebf8ff4 commit 525ffd7
Showing 1 changed file with 1 addition and 2 deletions.
3 changes: 1 addition & 2 deletions src/group_theory/subgroup/basic.lean
Expand Up @@ -2989,8 +2989,7 @@ instance sup_normal (H K : subgroup G) [hH : H.normal] [hK : K.normal] : (H ⊔

@[to_additive] instance normal_inf_normal (H K : subgroup G) [hH : H.normal] [hK : K.normal] :
(H ⊓ K).normal :=
{ conj_mem := λ n hmem g,
by { rw mem_inf at *, exact ⟨hH.conj_mem n hmem.1 g, hK.conj_mem n hmem.2 g⟩ } }
⟨λ n hmem g, ⟨hH.conj_mem n hmem.1 g, hK.conj_mem n hmem.2 g⟩⟩

@[to_additive] lemma subgroup_of_sup (A A' B : subgroup G) (hA : A ≤ B) (hA' : A' ≤ B) :
(A ⊔ A').subgroup_of B = A.subgroup_of B ⊔ A'.subgroup_of B :=
Expand Down

0 comments on commit 525ffd7

Please sign in to comment.