a4c0699e81
See issue #676 Add new test demonstrating why it is useful to have the old semantics for 'constructor'
6 lines
190 B
Text
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
|