Skip to content

Commit c29e7d7

Browse files
committed
fix: tighten imports
1 parent e321650 commit c29e7d7

File tree

1 file changed

+4
-4
lines changed

1 file changed

+4
-4
lines changed

src/Algebra/Construct/Centre/Group.agda

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -6,7 +6,7 @@
66

77
{-# OPTIONS --safe --cubical-compatible #-}
88

9-
open import Algebra.Bundles using (AbelianGroup; Group; RawGroup)
9+
open import Algebra.Bundles using (AbelianGroup; Group)
1010

1111
module Algebra.Construct.Centre.Group {c ℓ} (G : Group c ℓ) where
1212

@@ -36,7 +36,7 @@ private
3636

3737
open Carrier using (commuter; commutes)
3838

39-
_≈_ : Rel Carrier _
39+
_≈_ : Rel Carrier
4040
_≈_ = G._≈_ on commuter
4141

4242
_∙_ : Op₂ Carrier
@@ -74,7 +74,7 @@ private
7474
∙-comm : Commutative _≈_ _∙_
7575
∙-comm g h = commutes g $ commuter h
7676

77-
centre : NormalSubgroup _ _
77+
centre : NormalSubgroup (c ⊔ ℓ) ℓ
7878
centre = record
7979
{ subgroup = record
8080
{ domain = record
@@ -110,7 +110,7 @@ private
110110

111111
open NormalSubgroup centre public
112112

113-
abelianGroup : AbelianGroup _ _
113+
abelianGroup : AbelianGroup (c ⊔ ℓ) ℓ
114114
abelianGroup = record
115115
{ isAbelianGroup = record
116116
{ isGroup = isGroup

0 commit comments

Comments
 (0)