2015-02-11 20:49:27 +00:00
|
|
|
|
protected_test.lean:2:8: error: unknown identifier 'induction_on'
|
|
|
|
|
protected_test.lean:3:8: error: unknown identifier 'rec_on'
|
|
|
|
|
nat.induction_on : ∀ (n : ℕ), ?C 0 → (∀ (a : ℕ), ?C a → ?C (succ a)) → ?C n
|
2015-10-14 01:35:16 +00:00
|
|
|
|
le.rec_on : le ?a ?a_1 → ?C ?a → (∀ {b : ℕ}, le ?a b → ?C b → ?C (succ b)) → ?C ?a_1
|
|
|
|
|
le.rec_on : le ?a ?a_1 → ?C ?a → (∀ {b : ℕ}, le ?a b → ?C b → ?C (succ b)) → ?C ?a_1
|
2015-02-11 20:49:27 +00:00
|
|
|
|
protected_test.lean:8:10: error: unknown identifier 'rec_on'
|
2015-10-14 01:35:16 +00:00
|
|
|
|
le.rec_on : le ?a ?a_1 → ?C ?a → (∀ {b : ℕ}, le ?a b → ?C b → ?C (succ b)) → ?C ?a_1
|