@@ -42,7 +42,7 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
42
42
open FunctionDefinitions _≈₁_ _≈₂_
43
43
open FunctionStructures _≈₁_ _≈₂_
44
44
45
- record Injection : Set (a ⊔ b ⊔ suc ( ℓ₁ ⊔ ℓ₂) ) where
45
+ record Injection : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
46
46
field
47
47
f : A → B
48
48
cong : f Preserves _≈₁_ ⟶ _≈₂_
@@ -63,7 +63,7 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
63
63
; injective = injective
64
64
}
65
65
66
- record Surjection : Set (a ⊔ b ⊔ suc ( ℓ₁ ⊔ ℓ₂) ) where
66
+ record Surjection : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
67
67
field
68
68
f : A → B
69
69
cong : f Preserves _≈₁_ ⟶ _≈₂_
@@ -85,7 +85,7 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
85
85
}
86
86
87
87
88
- record Bijection : Set (a ⊔ b ⊔ suc ( ℓ₁ ⊔ ℓ₂) ) where
88
+ record Bijection : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
89
89
field
90
90
f : A → B
91
91
cong : f Preserves _≈₁_ ⟶ _≈₂_
@@ -121,15 +121,15 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
121
121
open IsBijection isBijection public using (module Eq₁ ; module Eq₂ )
122
122
123
123
124
- record Equivalence : Set (a ⊔ b ⊔ suc ( ℓ₁ ⊔ ℓ₂) ) where
124
+ record Equivalence : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
125
125
field
126
126
f : A → B
127
127
g : B → A
128
128
cong₁ : f Preserves _≈₁_ ⟶ _≈₂_
129
129
cong₂ : g Preserves _≈₂_ ⟶ _≈₁_
130
130
131
131
132
- record LeftInverse : Set (a ⊔ b ⊔ suc ( ℓ₁ ⊔ ℓ₂) ) where
132
+ record LeftInverse : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
133
133
field
134
134
f : A → B
135
135
g : B → A
@@ -160,7 +160,7 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
160
160
}
161
161
162
162
163
- record RightInverse : Set (a ⊔ b ⊔ suc ( ℓ₁ ⊔ ℓ₂) ) where
163
+ record RightInverse : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
164
164
field
165
165
f : A → B
166
166
g : B → A
@@ -189,7 +189,7 @@ module _ (From : Setoid a ℓ₁) (To : Setoid b ℓ₂) where
189
189
}
190
190
191
191
192
- record Inverse : Set (a ⊔ b ⊔ suc ( ℓ₁ ⊔ ℓ₂) ) where
192
+ record Inverse : Set (a ⊔ b ⊔ ℓ₁ ⊔ ℓ₂) where
193
193
field
194
194
f : A → B
195
195
f⁻¹ : B → A
0 commit comments