mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-13 17:25:29 +03:00
27 lines
413 B
Idris
27 lines
413 B
Idris
infixr 5 ::
|
|
|
|
export
|
|
data List a = Nil | (::) a (List a)
|
|
export
|
|
data Nat = Z | S Nat
|
|
|
|
export
|
|
data Vect : Type -> Type where
|
|
export
|
|
data Set : Type -> Type where
|
|
|
|
namespace Vect
|
|
export
|
|
toList : Vect a -> List a
|
|
export
|
|
fromList : List a -> Vect a
|
|
|
|
namespace Set
|
|
export
|
|
toList : Set a -> List a
|
|
export
|
|
fromList : List a -> Set a
|
|
|
|
keepUnique : List b -> List b
|
|
keepUnique {b} xs = toList (fromList xs)
|