definition test.foo.prf [irreducible] : ∀ (x : ℕ), 0 < succ (succ x) := λ (x : ℕ), lt.step (zero_lt_succ x) definition test.bla : ℕ → ℕ := λ (a : ℕ), foo (succ (succ a)) (foo.prf a) definition test.bla : ℕ → ℕ := λ (a : ℕ), test.foo (succ (succ a)) (test.foo.prf a) definition test.foo.prf : ∀ (x : ℕ), 0 < succ (succ x) := λ (x : ℕ), lt.step (zero_lt_succ x)