annotate 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
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
rev   line source
6
4bf00f7ba825 add description of agda
soto@cr.ie.u-ryukyu.ac.jp
parents:
diff changeset
1 data ℕ : Set where
4bf00f7ba825 add description of agda
soto@cr.ie.u-ryukyu.ac.jp
parents:
diff changeset
2 zero : ℕ
4bf00f7ba825 add description of agda
soto@cr.ie.u-ryukyu.ac.jp
parents:
diff changeset
3 suc : (n : ℕ) → ℕ