main.agda 321 B

12345678910111213
  1. module main where
  2. open import Not-named-according-to-the-Haskell-lexical-syntax
  3. main = return Not-named-according-to-the-Haskell-lexical-syntax.unit
  4. -- The following code once triggered an MAlonzo bug resulting in the
  5. -- error message "Panic: ... no such name main.M.d".
  6. module M where
  7. data D : Set where
  8. d : D