TheHoTTGame/0Trinitarianism/Preambles/P4.agda
2021-10-30 19:02:51 +01:00

6 lines
237 B
Agda

module 0Trinitarianism.Preambles.P4 where
open import Cubical.Foundations.Prelude using
( Level ; Type ; _≡_ ; J ; JRefl ; refl ; i1 ; i0 ; I ; cong) public
open import Cubical.Foundations.Isomorphism renaming (Iso to _≅_) public