Skip to content

Commit

Permalink
chore(Normed/../AddTorsor): improve readability (#9213)
Browse files Browse the repository at this point in the history
Pass more arguments to `choose!`
to avoid using projections later in the proof.
  • Loading branch information
urkud committed Dec 22, 2023
1 parent 83012aa commit 1462ef7
Showing 1 changed file with 4 additions and 4 deletions.
8 changes: 4 additions & 4 deletions Mathlib/Analysis/Normed/Group/AddTorsor.lean
Expand Up @@ -326,11 +326,11 @@ theorem IsClosed.vadd_right_of_isCompact {s : Set V} {t : Set P} (hs : IsClosed
-- This result is still true for any `AddTorsor` where `-ᵥ` is continuous,
-- but we don't yet have a nice way to state it.
refine IsSeqClosed.isClosed (fun u p husv hup ↦ ?_)
choose! a v hav using husv
rcases ht.isSeqCompact fun n ↦ (hav n).2.1 with ⟨q, hqt, φ, φ_mono, hφq⟩
choose! a v ha hv hav using husv
rcases ht.isSeqCompact hv with ⟨q, hqt, φ, φ_mono, hφq⟩
refine ⟨p -ᵥ q, q, hs.mem_of_tendsto ((hup.comp φ_mono.tendsto_atTop).vsub hφq)
(eventually_of_forall fun n ↦ ?_), hqt, vsub_vadd _ _⟩
convert (hav (φ n)).1 using 1
exact (eq_vadd_iff_vsub_eq _ _ _).mp (hav (φ n)).2.2.symm
convert ha (φ n) using 1
exact (eq_vadd_iff_vsub_eq _ _ _).mp (hav (φ n)).symm

end Pointwise

0 comments on commit 1462ef7

Please sign in to comment.