{-# OPTIONS --safe --warning=error --without-K #-} open import LogicalFormulae open import Orders open import Setoids.Setoids open import Functions open import Agda.Primitive using (Level; lzero; lsuc; _⊔_) module Setoids.Orders where record SetoidPartialOrder {a b c : _} {A : Set a} (S : Setoid {a} {b} A) (_<_ : Rel {a} {c} A) : Set (a ⊔ b ⊔ c) where open Setoid S field