2015-10-13 22:39:03 +00:00
|
|
|
open nat
|
|
|
|
|
2015-04-30 20:36:43 +00:00
|
|
|
example (a b : nat) (h : false) : a = b :=
|
|
|
|
by contradiction
|
|
|
|
|
|
|
|
example : ∀ (a b : nat), false → a = b :=
|
|
|
|
by contradiction
|
|
|
|
|
2015-10-13 22:39:03 +00:00
|
|
|
example : ∀ (a b : nat), (0:nat) = 1 → a = b :=
|
2015-04-30 20:36:43 +00:00
|
|
|
by contradiction
|
|
|
|
|
|
|
|
definition id {A : Type} (a : A) := a
|
|
|
|
|
|
|
|
example : ∀ (a b : nat), id false → a = b :=
|
|
|
|
by contradiction
|
|
|
|
|
2015-10-13 22:39:03 +00:00
|
|
|
example : ∀ (a b : nat), id ((0:nat) = 1) → a = b :=
|
2015-04-30 20:36:43 +00:00
|
|
|
by contradiction
|