Skip to content

Commit

Permalink
feat: port GroupTheory.Subgroup.Pointwise (#1981)
Browse files Browse the repository at this point in the history
Co-authored-by: Johan Commelin <johan@commelin.net>
  • Loading branch information
urkud and jcommelin committed Feb 1, 2023
1 parent b937210 commit b746237
Show file tree
Hide file tree
Showing 3 changed files with 562 additions and 8 deletions.
1 change: 1 addition & 0 deletions Mathlib.lean
Expand Up @@ -622,6 +622,7 @@ import Mathlib.GroupTheory.Subgroup.Actions
import Mathlib.GroupTheory.Subgroup.Basic
import Mathlib.GroupTheory.Subgroup.Finite
import Mathlib.GroupTheory.Subgroup.MulOpposite
import Mathlib.GroupTheory.Subgroup.Pointwise
import Mathlib.GroupTheory.Subgroup.Saturated
import Mathlib.GroupTheory.Subgroup.Simple
import Mathlib.GroupTheory.Subgroup.Zpowers
Expand Down
12 changes: 4 additions & 8 deletions Mathlib/GroupTheory/GroupAction/ConjAct.lean
Expand Up @@ -50,17 +50,13 @@ open MulAction Subgroup

variable {M G G₀ R K}

instance [Group G] : Group (ConjAct G) :=
by delta ConjAct; infer_instance
instance [Group G] : Group (ConjAct G) := ‹Group G›

instance [DivInvMonoid G] : DivInvMonoid (ConjAct G) :=
by delta ConjAct; infer_instance
instance [DivInvMonoid G] : DivInvMonoid (ConjAct G) := ‹DivInvMonoid G›

instance [GroupWithZero G] : GroupWithZero (ConjAct G) :=
by delta ConjAct; infer_instance
instance [GroupWithZero G] : GroupWithZero (ConjAct G) := ‹GroupWithZero G›

instance [Fintype G] : Fintype (ConjAct G) :=
by delta ConjAct; infer_instance
instance [Fintype G] : Fintype (ConjAct G) := ‹Fintype G›

@[simp]
theorem card [Fintype G] : Fintype.card (ConjAct G) = Fintype.card G :=
Expand Down

0 comments on commit b746237

Please sign in to comment.