A RetroSearch Logo

Home - News ( United States | United Kingdom | Italy | Germany ) - Football scores

Search Query:

Showing content from https://agda.github.io/agda-stdlib/master/Data.Unit.Polymorphic.Base.html below:

Data.Unit.Polymorphic.Base

Data.Unit.Polymorphic.Base
------------------------------------------------------------------------
-- The Agda standard library
--
-- A universe polymorphic unit type, as a Lift of the Level 0 one.
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}

module Data.Unit.Polymorphic.Base where

open import Level using (Level; Lift; lift)
import Data.Unit.Base as 

------------------------------------------------------------------------
-- A unit type defined as a synonym

 : { : Level}  Set 
 {} = Lift  ⊤.⊤

tt : { : Level}   {}
tt = lift ⊤.tt

RetroSearch is an open source project built by @garambo | Open a GitHub Issue

Search and Browse the WWW like it's 1997 | Search results from DuckDuckGo

HTML: 3.2 | Encoding: UTF-8 | Version: 0.7.4