lean2/tests/lean/run/bquant.lean
Leonardo de Moura c6ebe9456e feat(library/data/nat): add "bounded" quantifiers
Later, we will add support for arbitrary well-founded relations
2014-12-13 15:42:38 -08:00

11 lines
252 B
Text

import data.nat.bquant
open nat
example : is_true (∀ x, x ≤ 4 → x ≠ 6) :=
trivial
example : is_false (∀ x, x ≤ 5 → ∀ y, y < x → y * y ≠ x) :=
trivial
example : is_true (∀ x, x < 5 → ∃ y, y ≤ x + 5 ∧ y = 2*x) :=
trivial