Issue2712.agda 486 B

1234567891011121314151617
  1. -- Andreas, 2017-08-23, issue #2712
  2. --
  3. -- GHC Pragmas like LANGUAGE have to appear at the top of the Haskell file.
  4. {-# OPTIONS --no-main #-} -- Recognized as pragma option since #2714
  5. module Issue2712 where
  6. {-# FOREIGN GHC {-# LANGUAGE TupleSections #-} #-}
  7. postulate
  8. Pair : (A B : Set) → Set
  9. pair : {A B : Set} → A → B → Pair A B
  10. {-# COMPILE GHC Pair = type (,) #-}
  11. {-# COMPILE GHC pair = \ _ _ a b -> (a,) b #-} -- Test the availability of TupleSections