2014-08-01 16:37:23 +00:00
|
|
|
|
import logic
|
2014-09-03 23:00:38 +00:00
|
|
|
|
open decidable
|
2014-09-05 01:41:06 +00:00
|
|
|
|
open eq
|
2014-07-25 06:43:40 +00:00
|
|
|
|
|
|
|
|
|
inductive nat : Type :=
|
2014-08-22 22:46:10 +00:00
|
|
|
|
zero : nat,
|
|
|
|
|
succ : nat → nat
|
2014-09-17 21:39:05 +00:00
|
|
|
|
definition refl := @eq.refl
|
2014-09-04 23:36:06 +00:00
|
|
|
|
namespace nat
|
2014-07-25 06:43:40 +00:00
|
|
|
|
|
2014-09-04 22:03:59 +00:00
|
|
|
|
definition pred (n : nat) := nat.rec zero (fun m x, m) n
|
2014-07-25 06:43:40 +00:00
|
|
|
|
theorem pred_zero : pred zero = zero := refl _
|
|
|
|
|
theorem pred_succ (n : nat) : pred (succ n) = n := refl _
|
|
|
|
|
|
|
|
|
|
theorem zero_or_succ (n : nat) : n = zero ∨ n = succ (pred n)
|
|
|
|
|
:= induction_on n
|
2014-09-04 23:36:06 +00:00
|
|
|
|
(or.intro_left _ (refl zero))
|
|
|
|
|
(take m IH, or.intro_right _
|
2014-08-20 22:49:44 +00:00
|
|
|
|
(show succ m = succ (pred (succ m)), from congr_arg succ (symm (pred_succ m))))
|
2014-07-25 06:43:40 +00:00
|
|
|
|
|
|
|
|
|
theorem zero_or_succ2 (n : nat) : n = zero ∨ n = succ (pred n)
|
|
|
|
|
:= @induction_on _ n
|
2014-09-04 23:36:06 +00:00
|
|
|
|
(or.intro_left _ (refl zero))
|
|
|
|
|
(take m IH, or.intro_right _
|
2014-08-20 22:49:44 +00:00
|
|
|
|
(show succ m = succ (pred (succ m)), from congr_arg succ (symm (pred_succ m))))
|
2014-09-04 23:36:06 +00:00
|
|
|
|
end nat
|