2014-01-25 18:56:49 +00:00
|
|
|
|
Set: pp::colors
|
|
|
|
|
Set: pp::unicode
|
|
|
|
|
Assumed: a
|
|
|
|
|
Assumed: b
|
|
|
|
|
Assumed: f
|
|
|
|
|
Assumed: g
|
|
|
|
|
λ x x2 : ℕ, (∀ y : ℕ, g y = x) → x > x2 + x
|
|
|
|
|
funext (λ x : ℕ,
|
|
|
|
|
funext (λ x2 : ℕ,
|
|
|
|
|
imp_congr
|
|
|
|
|
(refl (∀ y : ℕ, g y = x))
|
2014-01-26 00:54:42 +00:00
|
|
|
|
(λ C::4 : ∀ y : ℕ, g y = x,
|
|
|
|
|
congr (congr2 Nat::gt (C::4 (a + x + b))) (congr2 (Nat::add x2) (C::4 x)))))
|