Zulip Chat Archive

Stream: Is there code for X?

Topic: tendsto_inv₀_cobounded


Jireh Loreaux (Nov 06 2023 at 18:48):

I'm pretty sure we don't have this. Am I wrong? Feel free to golf.

import Mathlib.Analysis.Normed.Field.Basic

namespace Filter

open Bornology Topology

theorem tendsto_inv₀_cobounded (𝕜 : Type*) [NormedField 𝕜] :
    Tendsto (Inv.inv : 𝕜  𝕜) (cobounded 𝕜) (𝓝 0) := by
  rw [comap_norm_atTop, @NormedAddCommGroup.tendsto_nhds_zero]
  intro ε 
  filter_upwards [(atTop_basis.comap (‖·‖)).mem_of_mem (i := (ε / 2)⁻¹) (by trivial)] with x hx
  simp only [Set.mem_preimage, Set.mem_Ici] at hx
  rw [norm_inv, inv_lt (lt_of_lt_of_le (by positivity) hx) ]
  exact ((inv_lt_inv  (half_pos )).mpr <| half_lt_self ).trans_le hx

end Filter

Yury G. Kudryashov (Nov 07 2023 at 04:54):

We should add comap Inv.inv (𝓝[≠] 0) = cobounded k

Jireh Loreaux (Nov 07 2023 at 04:54):

Yes, I have that in my draft.

Jireh Loreaux (Nov 07 2023 at 04:54):

I'll PR shortly.

Jireh Loreaux (Nov 07 2023 at 07:59):

#8234

Yury G. Kudryashov (Nov 08 2023 at 02:52):

I added more lemmas, revived my old branch with (nhds a)⁻¹ = nhds a⁻¹, and made your PR depend on mine. If you prefer to merge the old version, then review my modifications, then feel free to revert your branch and merge the PR.

Yury G. Kudryashov (Nov 08 2023 at 03:02):

BTW, once this PR is merged (one way or another), I'm going to get rid of comap norm atTop.

Jireh Loreaux (Nov 08 2023 at 03:02):

Yeah, I was planning on that too, but if you want to that's fine.

Yury G. Kudryashov (Nov 08 2023 at 04:21):

I started in branch#YK-comap-norm-atTop


Last updated: Dec 20 2023 at 11:08 UTC