Skip to content

Commit

Permalink
chore(analysis/analytic/basic): golf (#12965)
Browse files Browse the repository at this point in the history
Golf a 1-line proof, drop an unneeded assumption.
  • Loading branch information
urkud committed Mar 28, 2022
1 parent 33afea8 commit 73a9c27
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/analysis/analytic/basic.lean
Expand Up @@ -666,9 +666,9 @@ protected lemma formal_multilinear_series.has_fpower_series_on_ball [complete_sp
r_pos := h,
has_sum := λ y hy, by { rw zero_add, exact p.has_sum hy } }

lemma has_fpower_series_on_ball.sum [complete_space F] (h : has_fpower_series_on_ball f p x r)
lemma has_fpower_series_on_ball.sum (h : has_fpower_series_on_ball f p x r)
{y : E} (hy : y ∈ emetric.ball (0 : E) r) : f (x + y) = p.sum y :=
(h.has_sum hy).unique (p.has_sum (lt_of_lt_of_le hy h.r_le))
(h.has_sum hy).tsum_eq.symm

/-- The sum of a converging power series is continuous in its disk of convergence. -/
protected lemma formal_multilinear_series.continuous_on [complete_space F] :
Expand Down

0 comments on commit 73a9c27

Please sign in to comment.