Skip to content

Commit 3cf4c3b

Browse files
committed
Cleanup imports
1 parent 314a175 commit 3cf4c3b

File tree

1 file changed

+7
-12
lines changed

1 file changed

+7
-12
lines changed

src/Relation/Nullary/Finite/Setoid.agda

Lines changed: 7 additions & 12 deletions
Original file line numberDiff line numberDiff line change
@@ -10,15 +10,10 @@ module Relation.Nullary.Finite.Setoid where
1010

1111
open import Data.Fin.Base using (Fin)
1212
open import Data.Nat.Base using (ℕ)
13-
open import Data.Product.Base as ×
14-
open import Data.Sum.Base as ⊎ using (_⊎_; inj₁; inj₂)
15-
open import Data.Unit using (⊤; tt)
16-
open import Function
17-
open import Level renaming (suc to lsuc)
18-
open import Relation.Binary using (Rel; Setoid; IsEquivalence)
19-
import Relation.Binary.Reasoning.Setoid as SetR
20-
import Relation.Binary.Construct.On as On
21-
open import Relation.Binary.PropositionalEquality as ≡ using (_≡_)
13+
open import Function.Bundles using (Injection; Surjection; Inverse)
14+
open import Level using (Level; _⊔_) renaming (suc to lsuc)
15+
open import Relation.Binary.Bundles using (Setoid)
16+
open import Relation.Binary.PropositionalEquality.Properties using (setoid)
2217

2318
private
2419
variable
@@ -27,17 +22,17 @@ private
2722
record StrictlyFinite (X : Setoid c ℓ) : Set (c ⊔ ℓ) where
2823
field
2924
size :
30-
inv : Inverse X (≡.setoid (Fin size))
25+
inv : Inverse X (setoid (Fin size))
3126

3227
record Subfinite (X : Setoid c ℓ) : Set (c ⊔ ℓ) where
3328
field
3429
size :
35-
inj : Injection X (≡.setoid (Fin size))
30+
inj : Injection X (setoid (Fin size))
3631

3732
record FinitelyEnumerable (X : Setoid c ℓ) : Set (c ⊔ ℓ) where
3833
field
3934
size :
40-
srj : Surjection (≡.setoid (Fin size)) X
35+
srj : Surjection (setoid (Fin size)) X
4136

4237
record InjectsIntoFinitelyEnumerable (X : Setoid c ℓ) c′ ℓ′
4338
: Set (c ⊔ ℓ ⊔ lsuc (c′ ⊔ ℓ′)) where

0 commit comments

Comments
 (0)