Zulip Chat Archive
Stream: new members
Topic: Variable in goal gets renamed
Wojtek Wawrów (Aug 31 2021 at 13:08):
Trying to solve the following tutorial exercise:
lemma near_cluster :
cluster_point u a → ∀ ε > 0, ∀ N, ∃ n ≥ N, |u n - a| ≤ ε :=
begin
I begin my solution with the following:
intros h_clust ε ε_pos N,
unfold cluster_point at h_clust,
cases h_clust with φ hφ,
cases hφ with hφ₁ hφ₂,
specialize hφ₂ ε ε_pos,
cases hφ₂ with N hN,
use φ N,
but after doing this, the goal gets rewritten to φ N ≥ N_1 ∧ ...
. Why did the N get rewritten to N_1? I am meaning for it to be the exact same value as the N I introduced above. Not quite sure how to proceed with this one.
Alex J. Best (Aug 31 2021 at 13:20):
You have two things in your context called N, one from the first line introducing N and one from the second to last doing cases cases hφ₂ with N hN
you get another, I'd suggest calling the second one M or something instead so that things don't get confusde
Wojtek Wawrów (Aug 31 2021 at 13:22):
Oh derp, didn't even realize. Thanks a lot
Last updated: Dec 20 2023 at 11:08 UTC