List.agda 305 B

1234567891011121314151617
  1. module List where
  2. open import Prelude
  3. open import Star
  4. [_] : Set -> Rel True
  5. [ A ] = \_ _ -> A
  6. List : Set -> Set
  7. List A = Star [ A ] _ _
  8. -- Actually there isn't really that much interesting stuff to be
  9. -- done for lists that isn't generic.
  10. {- Note that the "proofs" are the elements of the list. -}