mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-11-29 03:24:02 +03:00
15 lines
338 B
Idris
15 lines
338 B
Idris
import Data.Vect
|
|
|
|
distrL : a -> List b -> List (a, b)
|
|
distrL a = map (a,)
|
|
|
|
distrR : b -> List a -> List (a, b)
|
|
distrR b = map (, b)
|
|
|
|
-- closeVect : List (n ** Vect n Nat)
|
|
-- closeVect = map (** flip replicate 3) [0..10]
|
|
|
|
insert : List (Nat,Nat,Nat,Nat)
|
|
insert = map (\ f => f (the Nat 0) (the Nat 1))
|
|
[(,,2,3), (2,,,3), (2,3,,)]
|