CompilingQNamePats.agda 274 B

12345678910111213141516
  1. open import Common.Prelude
  2. open import Common.Reflection
  3. postulate
  4. X Y : Set
  5. isX : QName → Bool
  6. isX (quote X) = true
  7. isX _ = false
  8. main : IO Unit
  9. main = putStrLn ((if isX (quote X) then "yes" else "no") +S+
  10. (if isX (quote Y) then "yes" else "no"))