mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-08 21:38:40 +00:00
11 lines
231 B
Agda
11 lines
231 B
Agda
{-# OPTIONS --safe --warning=error --without-K #-}
|
||
|
||
open import LogicalFormulae
|
||
open import Numbers.Naturals.Definition
|
||
|
||
module Numbers.Integers.Definition where
|
||
|
||
data ℤ : Set where
|
||
nonneg : ℕ → ℤ
|
||
negSucc : ℕ → ℤ
|