view src/agda/Nat.agda @ 6:4bf00f7ba825

add description of agda
author soto@cr.ie.u-ryukyu.ac.jp
date Mon, 14 Sep 2020 02:58:14 +0900
parents
children
line wrap: on
line source

data ℕ : Set where
  zero : ℕ
  suc  : (n : ℕ) → ℕ