Progress towards UFDs (#88)

This commit is contained in:
Patrick Stevens
2019-12-08 11:18:39 +00:00
committed by GitHub
parent 99c38495ce
commit 33098e94b0
20 changed files with 462 additions and 253 deletions

18
Lists/Definition.agda Normal file
View 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)