mirror of
https://github.com/Smaug123/CubicalTutorial
synced 2025-10-08 17:28:44 +00:00
First commit
This commit is contained in:
13
Naturals.agda
Normal file
13
Naturals.agda
Normal file
@@ -0,0 +1,13 @@
|
||||
{-# OPTIONS --safe --warning=error --without-K #-}
|
||||
|
||||
module Naturals where
|
||||
|
||||
data ℕ : Set where
|
||||
zero : ℕ
|
||||
succ : ℕ → ℕ
|
||||
|
||||
{-# BUILTIN NATURAL ℕ #-}
|
||||
|
||||
_+N_ : ℕ → ℕ → ℕ
|
||||
zero +N b = b
|
||||
succ a +N b = succ (a +N b)
|
Reference in New Issue
Block a user