mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-19 10:08:42 +00:00
Progress towards UFDs (#88)
This commit is contained in:
18
Lists/Definition.agda
Normal file
18
Lists/Definition.agda
Normal file
@@ -0,0 +1,18 @@
|
||||
{-# OPTIONS --safe --warning=error --without-K #-}
|
||||
|
||||
open import LogicalFormulae
|
||||
open import Functions
|
||||
|
||||
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)
|
Reference in New Issue
Block a user