2014-01-05 20:05:08 +00:00
|
|
|
import Int.
|
2014-01-01 20:28:18 +00:00
|
|
|
|
2014-01-05 20:05:08 +00:00
|
|
|
namespace foo.
|
|
|
|
variable a : Nat.
|
|
|
|
definition b := a.
|
2014-01-06 03:10:21 +00:00
|
|
|
theorem T : a = b := refl a.
|
2014-01-05 20:05:08 +00:00
|
|
|
axiom H : b >= a.
|
|
|
|
namespace bla.
|
|
|
|
variables a c d : Int.
|
|
|
|
check a + b + c.
|
|
|
|
end.
|
|
|
|
end.
|
2014-01-01 20:28:18 +00:00
|
|
|
|
2014-01-05 20:05:08 +00:00
|
|
|
check foo::T.
|
|
|
|
check foo::H.
|
|
|
|
check foo::a.
|
|
|
|
check foo::bla::a.
|
2014-01-01 20:28:18 +00:00
|
|
|
|
2014-01-05 20:05:08 +00:00
|
|
|
end
|