We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent ebf1eed commit 7a7350eCopy full SHA for 7a7350e
src/Relation/Nullary/Finite/Setoid.agda
@@ -111,10 +111,9 @@ include-/ {X = X} R = record
111
open Setoid X
112
open EquivalenceRelation R
113
114
-record StrictlyFinite (X : Setoid c ℓ) : Set (c ⊔ ℓ) where
+record StronglyFinite (X : Setoid c ℓ) (n : ℕ) : Set (c ⊔ ℓ) where
115
field
116
- size : ℕ
117
- inv : Inverse X (≡.setoid (Fin size))
+ inv : Inverse X (≡.setoid (Fin n))
118
119
record Subfinite (X : Setoid c ℓ) : Set (c ⊔ ℓ) where
120
0 commit comments