TheHoTTGame/0Trinitarianism/Quest4Solutions.agda
2021-10-14 13:40:21 +01:00

8 lines
165 B
Agda

module 0Trinitarianism.Quest4Solutions where
open import Cubical.Foundations.Prelude
data _≣_ {A : Type} : (x y : A) Type where
rfl : (x : A) x x