Zulip Chat Archive
Stream: Is there code for X?
Topic: Z is discrete
Adam Topaz (Aug 07 2021 at 17:31):
Do we have a lemma approximately like the following?
import analysis.normed_space.basic
example (n : ℤ) : ∥ n ∥ < 1 → n = 0 := sorry
Ruben Van de Velde (Aug 07 2021 at 17:36):
example (n : ℤ) : ∥ n ∥ < 1 → n = 0 := by {
rw int.norm_eq_abs,
norm_cast,
exact int.eq_zero_iff_abs_lt_one.mp
}
Patrick Massot (Aug 07 2021 at 17:38):
maybe we should have a library_search_mod_cast
:wink:
Adam Topaz (Aug 07 2021 at 17:39):
thanks @Ruben Van de Velde !
Heather Macbeth (Aug 07 2021 at 18:44):
FWIW, I have found docs#int.tendsto_coe_cofinite to be a useful abstract formulation of "ℤ
is discrete":
/-- Under the coercion from `ℤ` to `ℝ`, inverse images of compact sets are finite. -/
lemma tendsto_coe_cofinite : tendsto (coe : ℤ → ℝ) cofinite (cocompact ℝ) :=
Kevin Buzzard (Aug 07 2021 at 18:49):
This is a lovely way of thinking about it! Actually it would look even nicer using ideals not filters because then the co-
prefixes would go
Last updated: Dec 20 2023 at 11:08 UTC