[Agda] Positive numbers
Nils Anders Danielsson
nad at Cs.Nott.AC.UK
Mon Mar 2 20:49:58 CET 2009
On 2009-03-02 18:04, J.Burton at brighton.ac.uk wrote:
> data N : Set where
> zero : N
> succ : N -> N
>
> data N+ : N -> Set where
> pos : forall {n : N} -> (succ n) -> N+
The problem is that succ n is not a type.
--
/NAD
This message has been checked for viruses but the contents of an attachment
may still contain software viruses, which could damage your computer system:
you are advised to perform your own checks. Email communications with the
University of Nottingham may be monitored as permitted by UK legislation.
More information about the Agda
mailing list