lean2/tests/lean/ns1.lean
Leonardo de Moura 935c2a03a3 feat(*): change name conventions for Lean builtin libraries
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-01-05 19:21:44 -08:00

19 lines
No EOL
265 B
Text

import Int.
namespace foo.
variable a : Nat.
definition b := a.
theorem T : a = b := refl a.
axiom H : b >= a.
namespace bla.
variables a c d : Int.
check a + b + c.
end.
end.
check foo::T.
check foo::H.
check foo::a.
check foo::bla::a.
end