Erased-cubical-Pattern-matching-Erased.agda 457 B

12345678910111213141516
  1. {-# OPTIONS --erased-cubical --save-metas #-}
  2. module Erased-cubical-Pattern-matching-Erased where
  3. open import Agda.Builtin.String
  4. open import Erased-cubical-Pattern-matching-Cubical
  5. -- If c₁ and c₂ are treated as erased, then f might be compiled to
  6. -- something akin to ⊥-elim. However, the main module uses
  7. -- --cubical, not --erased-cubical, so f should not be compiled in
  8. -- that way.
  9. f : D → String
  10. f c₁ = "Success\n"
  11. f c₂ = "Failure\n"