2014-12-13 23:36:35 +00:00
|
|
|
import data.nat.bquant
|
|
|
|
open nat
|
|
|
|
|
2015-10-13 22:39:03 +00:00
|
|
|
example : is_true (∀ x : nat, x ≤ 4 → x ≠ 6) :=
|
2014-12-13 23:36:35 +00:00
|
|
|
trivial
|
|
|
|
|
2015-10-13 22:39:03 +00:00
|
|
|
example : is_false (∀ x : nat, x ≤ 5 → ∀ y, y < x → y * y ≠ x) :=
|
2014-12-13 23:36:35 +00:00
|
|
|
trivial
|
|
|
|
|
2015-10-13 22:39:03 +00:00
|
|
|
example : is_true (∀ x : nat, x < 5 → ∃ y, y ≤ x + 5 ∧ y = 2*x) :=
|
2014-12-13 23:36:35 +00:00
|
|
|
trivial
|