Skip to content

Commit

Permalink
Merge pull request #331 from math-comp/rm_lemmas_20210201
Browse files Browse the repository at this point in the history
lemmas that made their way into mathcomp
  • Loading branch information
CohenCyril authored Feb 9, 2021
2 parents 31562ae + 04b7172 commit a21bb29
Show file tree
Hide file tree
Showing 2 changed files with 3 additions and 16 deletions.
2 changes: 2 additions & 0 deletions CHANGELOG_UNRELEASED.md
Original file line number Diff line number Diff line change
Expand Up @@ -65,6 +65,8 @@
+ `ball_le`
- in `classical_sets.v`, lemma `bigcapCU`

- in `sequences.v`, lemmas `ler_sum_nat`, `sumr_const_nat`

### Infrastructure

### Misc
17 changes: 1 addition & 16 deletions theories/sequences.v
Original file line number Diff line number Diff line change
Expand Up @@ -336,21 +336,6 @@ Lemma eq_sum_telescope (V : zmodType) (u_ : V ^nat) n :
u_ n = u_ 0%N + series (telescope u_) n.
Proof. by rewrite telescopeK/= addrC addrNK. Qed.

(* TODO: port to mathcomp *)
(* missing mathcomp lemmas *)
Lemma ler_sum_nat (R : numDomainType) (m n : nat) (F G : nat -> R) :
(forall i, (m <= i < n)%N -> (F i <= G i)%O) ->
(\sum_(m <= i < n) F i <= \sum_(m <= i < n) G i)%O.
Proof.
move=> leFG; rewrite big_nat_cond [in X in _ <= X]big_nat_cond.
by rewrite ler_sum// => i; rewrite andbT => /leFG.
Qed.

Lemma sumr_const_nat (V : zmodType) (m n : nat) (x : V) :
\sum_(n <= i < m) x = x *+ (m - n).
Proof. by rewrite big_const_nat; elim: (m - n)%N => //= k ->; rewrite mulrS. Qed.
(* end missing mathcomp lemmas *)

Section series_patched.

Variables (N : nat) (K : numFieldType) (V : normedModType K).
Expand Down Expand Up @@ -1201,7 +1186,7 @@ Qed.
Lemma ereal_limD (R : realType) (f g : nat -> {ereal R}) :
cvg f -> cvg g -> ~~ adde_undef (lim f) (lim g) ->
(lim (f \+ g) = lim f + lim g)%E.
Proof.
Proof.
move=> cf cg fg; apply/(@cvg_lim _ _ ((f \+ g)%E @ \oo)) => //=. (* BUG *)
exact: ereal_cvgD.
Qed.
Expand Down

0 comments on commit a21bb29

Please sign in to comment.