lean2/tests/lean/run/choice_ctx.lean
Leonardo de Moura 069f217215 fix(frontends/lean/elaborator): use full local context for metavariables due to coercions and overloads
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-08-05 17:21:21 -07:00

20 lines
324 B
Text

import data.nat.basic
using nat
set_option pp.coercion true
namespace foo
theorem trans {a b c : nat} (H1 : a = b) (H2 : b = c) : a = c :=
trans H1 H2
end
using foo
theorem tst (a b : nat) (H0 : b = a) (H : b = 0) : a = 0
:= have H1 : a = b, from symm H0,
trans H1 H
definition f (a b : nat) :=
let x := 3 in
a + x