------------------------------------------------------------------------ -- The Agda standard library -- -- Polymorphic versions of standard definitions in Relation.Unary ------------------------------------------------------------------------ {-# OPTIONS --cubical-compatible --safe #-} module Relation.Unary.Polymorphic where open import Data.Empty.Polymorphic using (⊥) open import Data.Unit.Polymorphic using (⊤) open import Level using (Level) open import Relation.Unary using (Pred) private variable a ℓ : Level A : Set a ------------------------------------------------------------------------ -- Special sets -- The empty set. ∅ : Pred A ℓ ∅ = λ _ → ⊥ -- The universal set. U : Pred A ℓ U = λ _ → ⊤
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