{-# OPTIONS --without-K #-} module Common.Unit where open import Agda.Builtin.Unit public renaming (⊤ to Unit; tt to unit)