12345678910111213141516171819202122232425262728293031323334353637383940414243444546 |
- module Introduction.Data.Parameterised where
- data Nat : Set where
- zero : Nat
- suc : Nat -> Nat
- data Bool : Set where
- false : Bool
- true : Bool
- data List (A : Set) : Set where
- nil : List A
- cons : A -> List A -> List A
- nilNat = nil {Nat}
- null : {A : Set} -> List A -> Bool
- null nil = true
- null (cons _ _) = false
|