{-# OPTIONS --safe #-}
module KUIP where

open import Agda.Primitive renaming (Set to 𝒰)
open import Agda.Builtin.Equality

UIP :  {} {A : 𝒰 } {x y : A} (p q : x  y)  p  q
UIP refl refl = refl