C.agda 288 B

123456789101112131415
  1. -- This module contains various line-ending characters in order
  2. -- to test that they don't affect module source hash calculation.
  3. module C where
  4. -- CR -- --
  5. -- LF --
  6. --
  7. -- CRLF --
  8. --
  9. -- LFCR --
  10. --
  11. -- FF -- --
  12. -- NEXT LINE --…--
  13. -- LINE SEPARATOR --
--
  14. -- PARAGRAPH SEPARATOR --
--