2014-01-05 20:05:08 +00:00
|
|
|
import Int.
|
|
|
|
variable a : Int
|
|
|
|
variable n : Nat
|
|
|
|
axiom H1 : a + a + a = 10
|
|
|
|
axiom H2 : a = n
|
2014-01-06 03:10:21 +00:00
|
|
|
theorem T : a + n + a = 10 := subst H1 H2
|
2014-01-06 05:45:31 +00:00
|
|
|
set::option pp::coercion true
|
|
|
|
set::option pp::notation false
|
|
|
|
set::option pp::implicit true
|
2014-01-05 20:05:08 +00:00
|
|
|
print environment 1.
|