1924b2884c
Preparation for major refactoring in the tactic framework.
6 lines
148 B
Text
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
|