------------------------------------------------------------------------
-- The Agda standard library
--
-- Level polymorphic Empty type
------------------------------------------------------------------------

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

module Data.Empty.Polymorphic where

open import Level

data  { : Level} : Set  where

⊥-elim :  {w } {Whatever : Set w}   {}  Whatever
⊥-elim ()