module Empty where

open import Equality
open import FunctionExtensionality
open import Level

data Ø { : Level} : Set  where

Ø-elim :
  { ℓ' : Level}
  {A : Set ℓ'}
   -----------
  Ø {}  A
Ø-elim ()

ØisProp :
  { : Level}
  {x y : Ø {}}
   -----------
  x  y
ØisProp {x = ()}

Øuniq :
  { ℓ' : Level}
  {A : Set ℓ'}
  (f g : Ø {}  A)
   ---------------
  f  g
Øuniq f g = funext  ())