mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-01 09:49:24 +03:00
Merge pull request #387 from LibreCybernetics/fix-export-vect
Make Applicative implementation of Vect n public export.
This commit is contained in:
commit
cec56561c6
@ -795,6 +795,7 @@ transpose (x :: xs) = helper x (transpose xs) -- = [| x :: xs |]
|
||||
--------------------------------------------------------------------------------
|
||||
-- These only work if the length is known at run time!
|
||||
|
||||
public export
|
||||
implementation {k : Nat} -> Applicative (Vect k) where
|
||||
pure = replicate _
|
||||
fs <*> vs = zipWith apply fs vs
|
||||
|
Loading…
Reference in New Issue
Block a user