Issue1624.agda 353 B

12345678910111213141516171819
  1. module Issue1624 where
  2. open import Common.Char
  3. open import Common.String
  4. open import Common.List
  5. test : List Char → String
  6. test ('0' ∷ ('x' ∷ xs)) = "x"
  7. test ('0' ∷ ('b' ∷ xs)) = "b"
  8. test xs = "f"
  9. open import Common.IO
  10. open import Common.Unit
  11. main : IO Unit
  12. main = putStr (test x)
  13. where x = '0' ∷ ('x' ∷ ('1' ∷ []))