lean2/tests/lean/subst_bug.lean
2015-06-12 12:11:44 -07:00

14 lines
276 B
Text

example (f : nat → nat) (a b : nat) : f a = a → f (f a) = a :=
begin
intro h₁,
subst h₁ -- ERROR
end
open nat
example (f : nat → nat) (a b : nat) : f a = a → a = 0 → f (f a) = a :=
begin
intro h₁ h₂,
subst a, -- should use h₂
rewrite +h₁
end