lean2/tests/lean/unfold_rec.lean.expected.out
Leonardo de Moura a9515ac7a4 feat(library/tactic/rewrite_tactic): try to fold nested recursive applications after unfolding a recursive function
See issue #692.
The implementation still has some rough spots.
It is not clear what the right semantic is.
Moreover, the folds in e_closure could not be eliminated automatically.
2015-07-08 21:19:18 -04:00

20 lines
625 B
Text
Raw Blame History

This file contains ambiguous Unicode characters

This file contains Unicode characters that might be confused with other characters. If you think that this is intentional, you can safely ignore this warning. Use the Escape button to reveal them.

unfold_rec.lean:11:2: proof state
n m :
⊢ succ (succ n + m) = succ (succ (n + m))
unfold_rec.lean:24:2: proof state
n m :
⊢ succ (n + succ m) = succ (succ (n + m))
unfold_rec.lean:39:2: proof state
fibgt0 : ∀ (b n c : ), fib b n c > 0,
b m c :
⊢ fib b m c + fib b (succ m) c > 0
unfold_rec.lean:48:2: proof state
A : Type,
B : Type,
unzip_zip : ∀ {n : } (v₁ : vector A n) (v₂ : vector B n), unzip (zip v₁ v₂) = (v₁, v₂),
m : ,
a : A,
va : vector A m,
b : B,
vb : vector B m
⊢ (a :: prod.pr1 (unzip (zip va vb)), b :: prod.pr2 (unzip (zip va vb))) = (a :: va, b :: vb)