NakedEllipsisWeirdError.agda 336 B

1234567891011121314151617
  1. -- Andreas, 2019-08-10, weird error for naked ellipsis
  2. ...
  3. -- Error (weird):
  4. -- Missing type signature for left hand side ...
  5. -- when scope checking the declaration
  6. -- ...
  7. -- When following the suggestion to give a type signature,
  8. --
  9. -- ... : Set
  10. --
  11. -- Agda says:
  12. -- The ellipsis ... cannot have a type signature
  13. -- <EOF><ERROR>