mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-19 01:01:59 +03:00
Typo fix in Data/Vect/Properties/Fin.idr
This commit is contained in:
parent
809319fe8f
commit
e4337c118b
@ -35,7 +35,7 @@ finToElem {n } xs i with (finNonEmpty xs $ finNonZero i)
|
||||
finToElem {n = S n} (x :: xs) FZ | IsNonEmpty = Here
|
||||
finToElem {n = S n} (x :: xs) (FS i) | IsNonEmpty = There (finToElem xs i)
|
||||
|
||||
||| Analogus to `indexNaturality`, but morhisms can (irrelevantly) know the context
|
||||
||| Analogus to `indexNaturality`, but morphisms can (irrelevantly) know the context
|
||||
export
|
||||
indexNaturalityWithElem : (i : Fin n) -> (xs : Vect n a) -> (f : (x : a) -> (0 pos : x `Elem` xs) -> b)
|
||||
-> index i (mapWithElem xs f) = f (index i xs) (finToElem xs i)
|
||||
|
Loading…
Reference in New Issue
Block a user