Skip to content

Commit

Permalink
closed subgroup
Browse files Browse the repository at this point in the history
  • Loading branch information
zjj committed Aug 15, 2024
1 parent d8ab250 commit fd28b26
Showing 1 changed file with 10 additions and 0 deletions.
10 changes: 10 additions & 0 deletions BrauerGroup/Profinite/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -63,6 +63,8 @@ instance : CoeSort ProfiniteGrp (Type u) where

instance (G : ProfiniteGrp) : Group G := G.group

instance (G : ProfiniteGrp) : TopologicalGroup G := G.topologicalGroup

def of (G : Type u) [Group G] [TopologicalSpace G] [TopologicalGroup G]
[CompactSpace G] [TotallyDisconnectedSpace G] : ProfiniteGrp where
toCompHaus :=
Expand Down Expand Up @@ -134,6 +136,14 @@ def ofFiniteGrp (G : FiniteGrp) : ProfiniteGrp :=
letI : TopologicalGroup G := {}
of G

def ofClosedSubgroup {G : ProfiniteGrp}
(H : Subgroup G) (hH : IsClosed (H : Set G)) : ProfiniteGrp :=
letI : CompactSpace H := ClosedEmbedding.compactSpace (f := H.subtype)
{ induced := rfl
inj := H.subtype_injective
isClosed_range := by simpa }
of H

section

variable {J : Type v} [Category J] (F : J ⥤ FiniteGrp)
Expand Down

0 comments on commit fd28b26

Please sign in to comment.