Irrelevance.agda 191 B

1234567891011
  1. -- Andreas, 2012-01-12
  2. module Common.Irrelevance where
  3. open import Common.Level
  4. record Squash {a}(A : Set a) : Set a where
  5. constructor squash
  6. field
  7. .unsquash : A
  8. open Squash public