Skip to content

Commit

Permalink
not_near_at_leftP
Browse files Browse the repository at this point in the history
  • Loading branch information
IshiguroYoshihiro committed May 9, 2024
1 parent ccbfa1f commit d874edb
Show file tree
Hide file tree
Showing 2 changed files with 13 additions and 0 deletions.
3 changes: 3 additions & 0 deletions CHANGELOG_UNRELEASED.md
Original file line number Diff line number Diff line change
Expand Up @@ -31,6 +31,9 @@
+ lemmas `total_variation_nondecreasing`, `total_variation_bounded_variation`
- new file `theories/all_analysis.v`

- in `normedtype.v`:
+ lemma `not_near_at_leftP`

### Changed

- in `forms.v`:
Expand Down
10 changes: 10 additions & 0 deletions theories/normedtype.v
Original file line number Diff line number Diff line change
Expand Up @@ -1308,6 +1308,16 @@ apply: contrapT; apply: pePf; apply/andP; split.
- by near: t; apply: nbhs_right_lt; rewrite ltrDl.
Unshelve. all: by end_near. Qed.

Lemma not_near_at_leftP T (f : R -> T) (p : R) (P : pred T) :
~ (\forall x \near p^'-, P (f x)) ->
forall e : {posnum R}, exists2 x : R, p - e%:num < x < p & ~ P (f x).
Proof.
move=> pPf e; apply: contrapT => /forallPNP pePf; apply: pPf; near=> t.
apply: contrapT; apply: pePf; apply/andP; split.
- by near: t; apply: nbhs_left_gt; rewrite ltrBlDr ltrDl.
- by near: t; exact: nbhs_left_lt.
Unshelve. all: by end_near. Qed.

Lemma withinN (A : set R) a :
within A (nbhs (- a)) = - x @[x --> within (-%R @` A) (nbhs a)].
Proof.
Expand Down

0 comments on commit d874edb

Please sign in to comment.