{-# OPTIONS --safe --warning=error --without-K #-} open import Agda.Primitive using (Level; lzero; lsuc; _⊔_) open import LogicalFormulae open import Functions open import Orders.Total.Definition module Orders.Total.Lemmas {a b : _} {A : Set a} (order : TotalOrder A {b}) where open TotalOrder order equivMin : {x y : A} → (x < y) → min x y ≡ x equivMin {x} {y} x