16 lines
268 B
Agda
16 lines
268 B
Agda
module Trinitarianism.Quest1 where
|
||
|
||
open import Trinitarianism.Preambles.P1
|
||
|
||
isEven : ℕ → Type
|
||
isEven n = {!!}
|
||
|
||
{-
|
||
This is a comment block.
|
||
Remove this comment block and formulate
|
||
'there exists an even natural' here.
|
||
-}
|
||
|
||
div2 : Σ ℕ isEven → ℕ
|
||
div2 x = {!!}
|