Issue3965.agda 469 B

123456789101112131415161718192021
  1. open import Agda.Builtin.Nat
  2. f : Nat → Nat
  3. f 0 = zero
  4. f 0 = 0 -- All -- But Only
  5. f (suc n) = n -- These
  6. f 0 = 0 -- Lines -- These Two
  7. -- Used to be highlighted -- Should be!
  8. g : Nat → Nat
  9. g 0 = zero
  10. g 0 -- The highlihting should still
  11. = 0 -- span multiple lines if the clause does
  12. g (suc n) = n
  13. g 0 -- Even
  14. -- With
  15. -- A Lot
  16. = 0 -- Of Empty Lines in between