lean2/tests/lean/run/blast_meta.lean
Leonardo de Moura 9935cbc3d7 feat(library/blast/blast): communicate assigned metavariables back to tactic framework
We need this feature to be able to solve (input) goals containing
metavariables using blast.
See new test for example.
2016-01-02 20:05:44 -08:00

13 lines
235 B
Text

constant p : nat → nat → Prop
constant p_trans : ∀ a b c, p a b → p b c → p a c
definition lemma1 (a b c d : nat) : a = d → p b c → p a b → p a c :=
begin
intros,
apply p_trans,
blast,
blast
end
print lemma1