mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-12 07:08:40 +00:00
17 lines
352 B
Agda
17 lines
352 B
Agda
{-# OPTIONS --safe --warning=error --without-K #-}
|
|
|
|
|
|
module Lists.Definition {a : _} where
|
|
|
|
data List (A : Set a) : Set a where
|
|
[] : List A
|
|
_::_ : (x : A) (xs : List A) → List A
|
|
infixr 10 _::_
|
|
|
|
[_] : {A : Set a} → (a : A) → List A
|
|
[ a ] = a :: []
|
|
|
|
_++_ : {A : Set a} → List A → List A → List A
|
|
[] ++ m = m
|
|
(x :: l) ++ m = x :: (l ++ m)
|