Issue1430.agda 154 B

1234567891011
  1. -- Andreas, 2020-05-16, issue #4649
  2. -- Allow --safe flag in -I mode
  3. {-# OPTIONS --safe #-}
  4. data Unit : Set where
  5. unit : Unit
  6. test : Unit
  7. test = {!!}