Issue1496.agda 267 B

12345678910111213
  1. module Issue1496 where
  2. open import Common.Unit
  3. open import Common.String
  4. open import Common.Char
  5. open import Common.List
  6. open import Common.IO
  7. -- Agda infers that the "a" level argument to return has to be
  8. -- Agda.Primitive.lzero.
  9. main : IO Unit
  10. main = return unit