{-# OPTIONS --safe --warning=error --without-K #-} open import Agda.Primitive using (Level; lzero; lsuc; _⊔_) open import LogicalFormulae open import Functions module Orders where record PartialOrder {a b : _} (carrier : Set a) : Set (a ⊔ lsuc b) where field _<_ : Rel {a} {b} carrier irreflexive : {x : carrier} → (x < x) → False