Issue3898.agda 343 B

1234567891011121314151617
  1. {-# OPTIONS -v tc.force:60 #-}
  2. open import Agda.Builtin.Nat
  3. open import Agda.Builtin.List
  4. module _ {a} {A : Set a} where
  5. [_] : A → List A
  6. [ x ] = x ∷ []
  7. data FSet : List A → Set a where
  8. sg : (x : A) → FSet [ x ]
  9. -- ^ should be forced
  10. HOLE : Set
  11. HOLE = {!!} -- just to force make bugs to look at the output