Skip to content

Commit

Permalink
fixes #1473 (#1474)
Browse files Browse the repository at this point in the history
  • Loading branch information
affeldt-aist authored Feb 12, 2025
1 parent 7fda14e commit 7705e58
Show file tree
Hide file tree
Showing 3 changed files with 27 additions and 3 deletions.
6 changes: 6 additions & 0 deletions CHANGELOG_UNRELEASED.md
Original file line number Diff line number Diff line change
Expand Up @@ -97,6 +97,9 @@
+ module `gauss_integral_proof`
+ lemma `integral0y_gauss`

- in `normedtype.v`:
+ lemmas `ninfty`, `cvgy_compNP`

### Changed

- in `lebesgue_integral.v`
Expand All @@ -120,6 +123,9 @@
- in file `separation_axioms.v`, updated `discrete_hausdorff`, and
`discrete_zero_dimension` to take a `discreteTopologicalType`.

- in `normedtype.v`:
+ lemma `cvgyNP` renamed to `cvgNy_compN` and generalized

### Renamed

- in `measure.v`
Expand Down
22 changes: 20 additions & 2 deletions theories/normedtype.v
Original file line number Diff line number Diff line change
Expand Up @@ -387,6 +387,14 @@ apply/seteqP; split => [A [M [Mreal MA]]|A [M [Mreal MA]]].
by exists (- M); rewrite ?realN; split=> // x; rewrite ltrNr => /MA.
Qed.

Lemma ninfty {R : numFieldType} : (- x : R)%R @[x --> +oo] = -oo.
Proof.
apply/seteqP; split => [A [M [Mreal MA]]|A [M [Mreal MA]]].
exists (- M); rewrite realN; split => // x.
by rewrite -ltrNr => /MA/=; rewrite opprK.
by exists (- M); rewrite ?realN; split=> // x; rewrite ltrNl => /MA.
Qed.

Section infty_nbhs_instances.
Context {R : numFieldType}.
Implicit Types r : R.
Expand Down Expand Up @@ -1476,13 +1484,23 @@ Proof.
by rewrite at_leftN -?fmap_comp; under [_ \o _]eq_fun => ? do rewrite /= opprK.
Qed.

Lemma cvgyNP {T : topologicalType} {R : numFieldType}
(f : R -> T) (l : T) :
Lemma cvgNy_compNP {T : topologicalType} {R : numFieldType} (f : R -> T)
(l : set_system T) :
f x @[x --> -oo] --> l <-> (f \o -%R) x @[x --> +oo] --> l.
Proof.
have f_opp : f =1 (fun x => (f \o -%R) (- x)) by move=> x; rewrite /comp opprK.
by rewrite (eq_cvg -oo _ f_opp) fmap_comp ninftyN.
Qed.
#[deprecated(since="mathcomp-analysis 1.9.0", note="renamed to `cvgNy_compNP`")]
Notation cvgyNP := cvgNy_compNP (only parsing).

Lemma cvgy_compNP {T : topologicalType} {R : numFieldType} (f : R -> T)
(l : set_system T) :
f x @[x --> +oo] --> l <-> (f \o -%R) x @[x --> -oo] --> l.
Proof.
have f_opp : f =1 (fun x => (f \o -%R) (- x)) by move=> x; rewrite /comp opprK.
by rewrite (eq_cvg +oo _ f_opp) fmap_comp ninfty.
Qed.

Section open_itv_subset.
Context {R : realType}.
Expand Down
2 changes: 1 addition & 1 deletion theories/realfun.v
Original file line number Diff line number Diff line change
Expand Up @@ -333,7 +333,7 @@ Lemma cvg_ninftyP (f : R -> R) (l : R) :
f x @[x --> -oo] --> l <->
forall u : R^nat, (u n @[n --> \oo] --> -oo) -> f (u n) @[n --> \oo] --> l.
Proof.
rewrite cvgyNP cvg_pinftyP/= (@bij_forall R^nat _ -%R)//.
rewrite cvgNy_compNP cvg_pinftyP/= (@bij_forall R^nat _ -%R)//.
have u_opp (u : R^nat) :
((- u) n @[n --> \oo] --> +oo) = (u n @[n --> \oo] --> -oo).
by rewrite propeqE cvgNry.
Expand Down

0 comments on commit 7705e58

Please sign in to comment.