{-# OPTIONS --without-K #-}

-- Agda-hott library.
-- Author: Mario Román

-- Empty.  The empty type, representing falsehood.

open import base.Universes

module base.Empty where

  -- A datatype without constructors is the empty type.
  data  {ℓᵢ} : Type ℓᵢ where

  -- Ex falso quodlibet
  exfalso : ∀{ ℓᵢ} {A : Type }   {ℓᵢ}  A
  exfalso ()

  -- Negation
  ¬ : ∀{}  Type   Type 
  ¬ A = (A   {lzero})