Skip to content

Commit

Permalink
rm redundant lemma
Browse files Browse the repository at this point in the history
  • Loading branch information
affeldt-aist committed Aug 6, 2024
1 parent 13800f6 commit 62b655e
Show file tree
Hide file tree
Showing 2 changed files with 6 additions and 13 deletions.
7 changes: 0 additions & 7 deletions classical/set_interval.v
Original file line number Diff line number Diff line change
Expand Up @@ -207,13 +207,6 @@ move=> /andP[]; rewrite lt_neqAle => /andP[xz zx ->].
by rewrite andbT; split => //; exact/nesym/eqP.
Qed.

Lemma subset_itv_oo_ccW x y u v : (u <= x)%O -> (y <= v)%O ->
`]x, y[ `<=` `[u, v].
Proof.
move=> ux yv; apply: (subset_trans _ (@subset_itv_oo_cc _ _ _ _)) => z/=.
by rewrite !in_itv/= => /andP[? zy]; rewrite (le_lt_trans ux) ?(lt_le_trans zy).
Qed.

End set_itv_porderType.
Arguments neitv {d T} _.

Expand Down
12 changes: 6 additions & 6 deletions theories/realfun.v
Original file line number Diff line number Diff line change
Expand Up @@ -386,11 +386,11 @@ Let nondecreasing_at_right_is_cvgrW f a b r : a < r -> r < b ->
Proof.
move=> ar rb ndf H; apply: nondecreasing_at_right_is_cvgr.
- near=> s => x y xrs yrs xy; rewrite ndf//.
+ by apply: subset_itv_oo_ccW xrs; exact/ltW.
+ by apply: subset_itv_oo_ccW yrs; exact/ltW.
+ by apply: subset_itvW xrs; exact/ltW.
+ by apply: subset_itvW yrs; exact/ltW.
- near=> x; exists (f r) => _ /= [s srx <-]; rewrite ndf//.
+ by apply: subset_itv_oo_cc; rewrite in_itv/= ar.
+ by apply: subset_itv_oo_ccW srx; exact/ltW.
+ by apply: subset_itvW srx; exact/ltW.
+ by move: srx; rewrite in_itv/= => /andP[/ltW].
Unshelve. all: by end_near. Qed.

Expand All @@ -399,10 +399,10 @@ Let nondecreasing_at_left_is_cvgrW f a b r : a < r -> r < b ->
Proof.
move=> ar rb ndf H; apply: nondecreasing_at_left_is_cvgr.
- near=> s => x y xrs yrs xy; rewrite ndf//.
+ by apply: subset_itv_oo_ccW xrs; exact/ltW.
+ by apply: subset_itv_oo_ccW yrs; exact/ltW.
+ by apply: subset_itvW xrs; exact/ltW.
+ by apply: subset_itvW yrs; exact/ltW.
- near=> x; exists (f r) => _ /= [s srx <-]; rewrite ndf//.
+ by apply: subset_itv_oo_ccW srx; exact/ltW.
+ by apply: subset_itvW srx; exact/ltW.
+ by apply: subset_itv_oo_cc; rewrite in_itv/= ar.
+ by move: srx; rewrite in_itv/= => /andP[_ /ltW].
Unshelve. all: by end_near. Qed.
Expand Down

0 comments on commit 62b655e

Please sign in to comment.