Skip to content

Commit b01c992

Browse files
committed
fix
1 parent 78c46f8 commit b01c992

File tree

2 files changed

+5
-40
lines changed

2 files changed

+5
-40
lines changed

CHANGELOG_UNRELEASED.md

Lines changed: 5 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -212,7 +212,7 @@
212212
- in `set_interval.v`:
213213
+ lemma `set_itv_splitU`
214214

215-
- in `normedtype.v`:
215+
- in `num_topology.v`:
216216
+ lemma `lt_nbhsr`
217217

218218
- in `realfun.v`:
@@ -255,6 +255,10 @@
255255
- in `Rstruct.v`
256256
+ instantiate `GRinv.inv` by `Rinv` instead of `Rinvx`
257257

258+
- moved from `normedtype.v` to `num_topology.v` and renamed:
259+
+ `nbhs_lt` -> `lt_nbhsl_lt`
260+
+ `nbhs_le` -> `lt_nbhsl_le`
261+
258262
### Renamed
259263

260264
- file `itv.v` to `interval_inference.v`
@@ -338,10 +342,6 @@
338342
+ `inum_min` -> `num_min`
339343
+ `inum_max` -> `num_max`
340344

341-
- in `normedtype.v`:
342-
+ `nbhs_lt` -> `lt_nbhsl_lt`
343-
+ `nbhs_le` -> `lt_nbhsl_le`
344-
345345
### Generalized
346346

347347
- in `sequences.v`,

theories/normedtype.v

Lines changed: 0 additions & 35 deletions
Original file line numberDiff line numberDiff line change
@@ -1198,41 +1198,6 @@ Arguments cvgr0_norm_le {_ _ _ F FF}.
11981198
#[global] Hint Extern 0 (is_true (`|?x| <= _)) => match goal with
11991199
H : x \is_near _ |- _ => near: x; exact: cvgr0_norm_le end : core.
12001200

1201-
Section nbhs_lt_le.
1202-
Context {R : numFieldType}.
1203-
Implicit Types x z : R.
1204-
1205-
Lemma lt_nbhsl_lt x z : x < z -> \forall y \near x, x <= y -> y < z.
1206-
Proof.
1207-
move=> xz; near=> y.
1208-
rewrite le_eqVlt => /predU1P[<-//|].
1209-
near: y; exists (z - x) => /=; first by rewrite subr_gt0.
1210-
move=> y/= /[swap] xy; rewrite ltr0_norm ?subr_lt0//.
1211-
by rewrite opprD addrC ltrBlDr subrK opprK.
1212-
Unshelve. all: by end_near. Qed.
1213-
1214-
Lemma lt_nbhsl_le x z : x < z -> \forall y \near x, x <= y -> y <= z.
1215-
Proof.
1216-
by move=> xz; apply: filterS (lt_nbhsl_lt xz) => y /[apply] /ltW.
1217-
Qed.
1218-
1219-
End nbhs_lt_le.
1220-
(*#[deprecated(since="mathcomp-analysis 1.9.0", note="use `lt_nbhsl_lt` instead")]
1221-
Notation nbhs_lt := lt_nbhsl_lt (only parsing).
1222-
#[deprecated(since="mathcomp-analysis 1.9.0", note="use `lt_nbhsl_le` instead")]
1223-
Notation nbhs_le := lt_nbhsl_le (only parsing).*)
1224-
1225-
Lemma lt_nbhsr {R : realFieldType} (a z : R) : a < z ->
1226-
\forall x \near z, a < x.
1227-
Proof.
1228-
rewrite -subr_gt0 => za0; exists (z - a) => //= u/=.
1229-
rewrite ltrBrDl addrC -ltrBrDl => /lt_le_trans; apply.
1230-
rewrite lerBlDl.
1231-
have [uz|uz] := leP u z.
1232-
by rewrite ger0_norm ?subr_ge0// subrK.
1233-
by rewrite ltr0_norm ?subr_lt0// opprB addrAC -lerBlDr opprK lerD// ?ltW.
1234-
Qed.
1235-
12361201
Section open_closed_sets.
12371202
(* TODO: duplicate theory within the subspace topology of Num.real
12381203
in a numDomainType *)

0 commit comments

Comments
 (0)