Skip to content

Commit 4c65e8a

Browse files
Reduce universe levels in Function.Bundles
1 parent 96049d0 commit 4c65e8a

File tree

1 file changed

+7
-7
lines changed

1 file changed

+7
-7
lines changed

src/Function/Bundles.agda

Lines changed: 7 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -42,7 +42,7 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
4242
open FunctionDefinitions _≈₁_ _≈₂_
4343
open FunctionStructures _≈₁_ _≈₂_
4444

45-
record Injection : Set (a ⊔ b ⊔ suc (ℓ₁ ⊔ ℓ₂)) where
45+
record Injection : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
4646
field
4747
f : A B
4848
cong : f Preserves _≈₁_ ⟶ _≈₂_
@@ -63,7 +63,7 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
6363
; injective = injective
6464
}
6565

66-
record Surjection : Set (a ⊔ b ⊔ suc (ℓ₁ ⊔ ℓ₂)) where
66+
record Surjection : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
6767
field
6868
f : A B
6969
cong : f Preserves _≈₁_ ⟶ _≈₂_
@@ -85,7 +85,7 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
8585
}
8686

8787

88-
record Bijection : Set (a ⊔ b ⊔ suc (ℓ₁ ⊔ ℓ₂)) where
88+
record Bijection : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
8989
field
9090
f : A B
9191
cong : f Preserves _≈₁_ ⟶ _≈₂_
@@ -121,15 +121,15 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
121121
open IsBijection isBijection public using (module Eq₁; module Eq₂)
122122

123123

124-
record Equivalence : Set (a ⊔ b ⊔ suc (ℓ₁ ⊔ ℓ₂)) where
124+
record Equivalence : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
125125
field
126126
f : A B
127127
g : B A
128128
cong₁ : f Preserves _≈₁_ ⟶ _≈₂_
129129
cong₂ : g Preserves _≈₂_ ⟶ _≈₁_
130130

131131

132-
record LeftInverse : Set (a ⊔ b ⊔ suc (ℓ₁ ⊔ ℓ₂)) where
132+
record LeftInverse : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
133133
field
134134
f : A B
135135
g : B A
@@ -160,7 +160,7 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
160160
}
161161

162162

163-
record RightInverse : Set (a ⊔ b ⊔ suc (ℓ₁ ⊔ ℓ₂)) where
163+
record RightInverse : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
164164
field
165165
f : A B
166166
g : B A
@@ -189,7 +189,7 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
189189
}
190190

191191

192-
record Inverse : Set (a ⊔ b ⊔ suc (ℓ₁ ⊔ ℓ₂)) where
192+
record Inverse : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
193193
field
194194
f : A B
195195
f⁻¹ : B A

0 commit comments

Comments
 (0)