lean2/tests/lean/run/eassumption.lean
Leonardo de Moura 1924b2884c refactor(library/tactic): remove 'append' and 'interleave' tacticals
Preparation for major refactoring in the tactic framework.
2016-02-24 16:02:16 -08:00

6 lines
148 B
Text

variable p : nat → Prop
variable q : nat → Prop
variables a b c : nat
example : p c → p b → q b → p a → ∃ x, p x ∧ q x :=
by blast