lean2/tests/lean/run/eassumption.lean
Leonardo de Moura a4c0699e81 feat(library/tactic/constructor_tactic): restore 'constructor' tactic old semantics, add 'fconstructor' tactic
See issue #676

Add new test demonstrating why it is useful to have the old semantics
for 'constructor'
2015-06-17 23:48:54 -07:00

6 lines
190 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 intros; repeat (constructor | eassumption); now