Skip to content

Commit

Permalink
near_in_itv_oy/yo/yy
Browse files Browse the repository at this point in the history
  • Loading branch information
IshiguroYoshihiro committed Oct 29, 2024
1 parent 57b7b2d commit d3b6809
Show file tree
Hide file tree
Showing 2 changed files with 39 additions and 1 deletion.
1 change: 1 addition & 0 deletions CHANGELOG_UNRELEASED.md
Original file line number Diff line number Diff line change
Expand Up @@ -56,6 +56,7 @@
`nbhs_one_point_compactification_weakE`,
`locally_compact_completely_regular`, and
`completely_regular_regular`.
+ new lemmas `near_in_itvoy`, `near_in_itvyo`, `near_in_itvyy`

### Changed

Expand Down
39 changes: 38 additions & 1 deletion theories/normedtype.v
Original file line number Diff line number Diff line change
Expand Up @@ -5336,10 +5336,47 @@ Lemma bound_itvE (R : numDomainType) (a b : R) :
(a \in `]-oo, a]).
Proof. by rewrite !(boundr_in_itv, boundl_in_itv). Qed.

Lemma near_in_itv {R : realFieldType} (a b : R) :
Section near_in_itv.
Context {R : realFieldType} (a b : R).

Lemma near_in_itv :
{in `]a, b[, forall y, \forall z \near y, z \in `]a, b[}.
Proof. exact: interval_open. Qed.

Lemma near_in_itvoy :
{in `]a, +oo[, forall y, \forall z \near y, z \in `]a, +oo[}.
Proof.
move=> x ax.
near=> z.
suff : z \in `]a, +oo[%classic by rewrite inE.
near: z.
rewrite near_nbhs.
apply: (@open_in_nearW _ _ `]a, +oo[%classic) => //.
by rewrite inE/=.
Unshelve. end_near. Qed.

Lemma near_in_itvyo :
{in `]-oo, b[, forall y, \forall z \near y, z \in `]-oo, b[}.
Proof.
move=> x xb.
near=> z.
suff : z \in `]-oo, b[%classic by rewrite inE.
near: z.
rewrite near_nbhs.
apply: (@open_in_nearW _ _ `]-oo, b[%classic) => //.
by rewrite inE/=.
Unshelve. end_near. Qed.

Lemma near_in_itvyy :
{in `]-oo, +oo[, forall y : R, \forall z \near y, z \in `]-oo, +oo[}.
Proof.
move=> x _.
rewrite -near_nbhs.
exact: nearW => //.
Qed.

End near_in_itv.

Lemma cvg_patch {R : realType} (f : R -> R^o) (a b : R) (x : R) : (a < b)%R ->
x \in `]a, b[ ->
f @ (x : subspace `[a, b]) --> f x ->
Expand Down

0 comments on commit d3b6809

Please sign in to comment.