File tree Expand file tree Collapse file tree 1 file changed +11
-4
lines changed Expand file tree Collapse file tree 1 file changed +11
-4
lines changed Original file line number Diff line number Diff line change @@ -10,19 +10,26 @@ open import Algebra.Bundles using (Group)
1010
1111module Algebra.NormalSubgroup {c ℓ} (G : Group c ℓ) where
1212
13+ open import Algebra.Definitions
1314open import Algebra.Construct.Sub.Group G using (Subgroup)
14- open import Data.Product.Base using (∃-syntax)
15+ open import Data.Product.Base using (∃-syntax; _,_ )
1516open import Level using (suc; _⊔_)
1617
1718private
1819 module G = Group G
1920
21+ -- every element of the subgroup commutes in G
22+ Normal : ∀ {c′ ℓ′} → Subgroup c′ ℓ′ → Set (c ⊔ ℓ ⊔ c′)
23+ Normal subgroup = ∀ n g → ∃[ n′ ] g G.∙ ι n G.≈ ι n′ G.∙ g
24+ where open Subgroup subgroup
25+
2026record NormalSubgroup c′ ℓ′ : Set (c ⊔ ℓ ⊔ suc (c′ ⊔ ℓ′)) where
2127 field
2228 subgroup : Subgroup c′ ℓ′
29+ normal : Normal subgroup
2330
2431 open Subgroup subgroup public
2532
26- field
27- -- every element of N commutes in G
28- normal : ∀ n g → ∃[ n′ ] g G.∙ ι n G.≈ ι n′ G.∙ g
33+ abelian⇒subgroup-normal : ∀ {c′ ℓ′} → Commutative G._≈_ G._∙_ → (subgroup : Subgroup c′ ℓ′) → Normal subgroup
34+ abelian⇒subgroup-normal ∙-comm subgroup n g = n , ∙-comm g (ι n)
35+ where open Subgroup subgroup
You can’t perform that action at this time.
0 commit comments