File tree Expand file tree Collapse file tree 1 file changed +9
-3
lines changed Expand file tree Collapse file tree 1 file changed +9
-3
lines changed Original file line number Diff line number Diff line change @@ -19,17 +19,23 @@ private
1919 module G = Group G
2020
2121-- every element of the subgroup commutes in G
22+ record IsNormal {c′ ℓ′} (subgroup : Subgroup c′ ℓ′) : Set (c ⊔ ℓ ⊔ c′) where
23+ open Subgroup subgroup
24+ field
25+ normal : ∀ n g → ∃[ n′ ] ι n′ G.∙ g G.≈ g G.∙ ι n
26+
2227Normal : ∀ {c′ ℓ′} → Subgroup c′ ℓ′ → Set (c ⊔ ℓ ⊔ c′)
2328Normal subgroup = ∀ n g → ∃[ n′ ] ι n′ G.∙ g G.≈ g G.∙ ι n
2429 where open Subgroup subgroup
2530
2631record NormalSubgroup c′ ℓ′ : Set (c ⊔ ℓ ⊔ suc (c′ ⊔ ℓ′)) where
2732 field
2833 subgroup : Subgroup c′ ℓ′
29- normal : Normal subgroup
34+ isNormal : IsNormal subgroup
3035
3136 open Subgroup subgroup public
37+ open IsNormal isNormal public
3238
33- abelian⇒subgroup-normal : ∀ {c′ ℓ′} → Commutative G._≈_ G._∙_ → (subgroup : Subgroup c′ ℓ′) → Normal subgroup
34- abelian⇒subgroup-normal ∙-comm subgroup n g = n , ∙-comm (ι n) g
39+ abelian⇒subgroup-normal : ∀ {c′ ℓ′} → Commutative G._≈_ G._∙_ → (subgroup : Subgroup c′ ℓ′) → IsNormal subgroup
40+ abelian⇒subgroup-normal ∙-comm subgroup = record { normal = λ n g → n , ∙-comm (ι n) g }
3541 where open Subgroup subgroup
You can’t perform that action at this time.
0 commit comments