Skip to content

Commit

Permalink
adapt to mc#1256
Browse files Browse the repository at this point in the history
  • Loading branch information
Tragicus committed Nov 25, 2024
1 parent 7c12c63 commit 2839d05
Show file tree
Hide file tree
Showing 3 changed files with 5 additions and 4 deletions.
2 changes: 1 addition & 1 deletion reals/constructive_ereal.v
Original file line number Diff line number Diff line change
Expand Up @@ -137,7 +137,7 @@ Definition er_map T T' (f : T -> T') (x : \bar T) : \bar T' :=
Lemma er_map_idfun T (x : \bar T) : er_map idfun x = x.
Proof. by case: x. Qed.

Definition fine {R : zmodType} x : R := if x is EFin v then v else 0.
Definition fine {R : zmodType} x : R := if x is EFin v then v else 0%R.

Section EqEReal.
Variable (R : eqType).
Expand Down
4 changes: 2 additions & 2 deletions theories/normedtype.v
Original file line number Diff line number Diff line change
Expand Up @@ -244,11 +244,11 @@ Proof.
apply/seteqP; split=> [A [e/= e0 reA]|_/= [A [e/= e0 reA <-]]].
exists (-%R @` A).
exists e => // x/= rxe xr; exists (- x)%R; rewrite ?opprK//.
by apply: reA; rewrite ?eqr_opp//= opprK addrC distrC.
by apply: reA; rewrite ?(@eqr_opp R)//= opprK addrC distrC.
rewrite image_comp (_ : _ \o _ = idfun) ?image_id// funeqE => x/=.
by rewrite opprK.
exists e => //= x/=; rewrite -opprD normrN => axe xa.
exists (- x)%R; rewrite ?opprK//; apply: reA; rewrite ?eqr_oppLR//=.
exists (- x)%R; rewrite ?opprK//; apply: reA; rewrite ?(@eqr_oppLR R)//=.
by rewrite opprK.
Qed.

Expand Down
3 changes: 2 additions & 1 deletion theories/showcase/summability.v
Original file line number Diff line number Diff line change
Expand Up @@ -35,8 +35,9 @@ apply: filter_fromT_filter; first by exists fset0.
by move=> A B /=; exists (A `|` B) => P /=; rewrite fsubUset => /andP[].
Qed.

Print Visibility.
Definition partial_sum {I : choiceType} {R : zmodType}
(x : I -> R) (A : {fset I}) : R := \sum_(i : A) x (val i).
(x : I -> R) (A : {fset I}) : R := (\sum_(i : A) x (val i))%R.

Definition sum (I : choiceType) {K : numDomainType} {R : normedModType K}
(x : I -> R) : R := lim (partial_sum x @ totally).
Expand Down

0 comments on commit 2839d05

Please sign in to comment.