13 lines
210 B
Agda
13 lines
210 B
Agda
|
||
module TheHoTTGame.Trinitarianism.AsProps.Quest0Preamble where
|
||
|
||
open import Cubical.Core.Everything hiding (_∨_) public
|
||
open import Cubical.Data.Nat public
|
||
|
||
private
|
||
postulate
|
||
u : Level
|
||
|
||
Prop = Type u
|
||
|