10 lines
174 B
Agda
10 lines
174 B
Agda
|
||
module Trinitarianism.Quest0Preamble where
|
||
|
||
open import Cubical.Core.Everything hiding (_∨_) public
|
||
open import Cubical.Data.Nat public
|
||
|
||
private
|
||
postulate
|
||
u : Level
|