mirror of
https://github.com/Smaug123/agdaproofs
synced 2025-10-13 15:48:39 +00:00
17 lines
323 B
Agda
17 lines
323 B
Agda
{-# OPTIONS --warning=error --safe --without-K #-}
|
||
|
||
open import LogicalFormulae
|
||
|
||
module Numbers.Naturals.Definition where
|
||
|
||
data ℕ : Set where
|
||
zero : ℕ
|
||
succ : ℕ → ℕ
|
||
|
||
infix 100 succ
|
||
|
||
{-# BUILTIN NATURAL ℕ #-}
|
||
|
||
succInjective : {a b : ℕ} → (succ a ≡ succ b) → a ≡ b
|
||
succInjective {a} {.a} refl = refl
|