lean2/tests/lean/run/blast_back1.lean

13 lines
201 B
Text
Raw Normal View History

constant r : nat → Prop
constant p : nat → Prop
definition q (a : nat) := p a
lemma rq [intro] : ∀ a, r a → q a :=
sorry
attribute q [reducible]
example (a : nat) : r a → p a :=
by blast