Zulip Chat Archive

Stream: new members

Topic: le_sub_iff_add_le error


Calle Sönne (Feb 22 2019 at 11:06):

I have following code, which gives an error on the last line:

lemma limit_start_irrelevant (a :   ) (k : ) (l : ) (h : M1P1.is_limit (λ n, a (n+k)) l) : M1P1.is_limit a l :=
begin
intros ε , cases h ε  with N H, use N + k, intros n Hn, simp only at H, rw le_sub_iff_add_le N k n at Hn,
end

Tactic state:

function expected at
  le_sub_iff_add_le
term has type
  ?m_3  ?m_4 - ?m_5  ?m_3 + ?m_5  ?m_4
state:
a :   ,
k : ,
l : ,
h : M1P1.is_limit (λ (n : ), a (n + k)) l,
ε : ,
 : ε > 0,
N n : ,
Hn : n  N + k,
H :  (n : ), n  N  |a (n + k) - l| < ε
 |a n - l| < ε

I can't seem to figure out what the problem is, subtracting naturals is fishy but lean seems to be complaining about something else. Any help would be appreciated :)

Mario Carneiro (Feb 22 2019 at 11:07):

you wrote le_sub_iff_add_le N k n but it takes no explicit arguments

Calle Sönne (Feb 22 2019 at 11:09):

Right, without arguments I get this error:

rewrite tactic failed, did not find instance of the pattern in the target expression
  _  ?m_5
state:
a :   ,
k : ,
l : ,
h : M1P1.is_limit (λ (n : ), a (n + k)) l,
ε : ,
 : ε > 0,
N n : ,
Hn : n  N + k,
H :  (n : ), n  N  |a (n + k) - l| < ε
 |a n - l| < ε

Do I need to "flip" the inequality? I thought both sides were treated as equal.

Kenny Lau (Feb 22 2019 at 11:13):

try erw

Mario Carneiro (Feb 22 2019 at 11:13):

try rw ge at Hn?

Kenny Lau (Feb 22 2019 at 11:13):

wait I know why

Kenny Lau (Feb 22 2019 at 11:13):

you're dealing with natural numbers.

Kenny Lau (Feb 22 2019 at 11:13):

:face_palm:

Mario Carneiro (Feb 22 2019 at 11:14):

There are similar theorems explicitly for nat

Mario Carneiro (Feb 22 2019 at 11:14):

you can't use the general theorem

Kenny Lau (Feb 22 2019 at 11:14):

but it still won't match the le with ge I guess

Kenny Lau (Feb 22 2019 at 11:14):

so you need to use erw or replace Hn := _

Mario Carneiro (Feb 22 2019 at 11:15):

I think you want replace Hn := nat.le_sub_right_of_add_le Hn

Calle Sönne (Feb 22 2019 at 11:18):

that worked. Thank you :)


Last updated: Dec 20 2023 at 11:08 UTC