Skip to content

Commit

Permalink
Port from signed to itv
Browse files Browse the repository at this point in the history
And deprecate signed.
  • Loading branch information
proux01 committed Nov 25, 2024
1 parent ce41c55 commit 89faa96
Show file tree
Hide file tree
Showing 37 changed files with 812 additions and 329 deletions.
2 changes: 2 additions & 0 deletions CHANGELOG_UNRELEASED.md
Original file line number Diff line number Diff line change
Expand Up @@ -56,6 +56,8 @@

### Deprecated

- file `signed.v` (use `itv.v` instead)

- in `itv.v`:
+ notation `%:inum` (use `%:num` instead)

Expand Down
2 changes: 1 addition & 1 deletion analysis_stdlib/Rstruct_topology.v
Original file line number Diff line number Diff line change
Expand Up @@ -12,7 +12,7 @@ From mathcomp Require Import archimedean.
From HB Require Import structures.
From mathcomp Require Import mathcomp_extra.
From mathcomp Require Import boolp classical_sets.
From mathcomp Require Import reals signed.
From mathcomp Require Import reals itv.
From mathcomp Require Import topology.
From mathcomp Require Export Rstruct.

Expand Down
4 changes: 2 additions & 2 deletions analysis_stdlib/showcase/uniform_bigO.v
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ From Coq Require Import Reals.
From Coq Require Import ssreflect ssrfun ssrbool.
From mathcomp Require Import ssrnat eqtype choice fintype bigop order ssralg ssrnum.
From mathcomp Require Import boolp reals Rstruct_topology ereal.
From mathcomp Require Import classical_sets signed topology normedtype landau.
From mathcomp Require Import classical_sets itv topology normedtype landau.

Set Implicit Arguments.
Unset Strict Implicit.
Expand Down Expand Up @@ -98,7 +98,7 @@ Proof.
move=> fOg; apply/Ouex_to_P; move: fOg => /eqOP [k [kreal hk]].
have /hk [Q [->]] : k < maxr 1 (k + 1) by rewrite lt_max ltrDl orbC ltr01.
move=> [R [[_/posnumP[e1] Re1] [_/posnumP[e2] Re2]] sRQ] fOg.
exists (minr e1%:num e2%:num) => //.
exists (minr e1%:num e2%:num); first by apply: gt0; exact: RbaseSymbolsImpl.R.
exists (maxr 1 (k + 1)); first by rewrite lt_max ltr01.
move=> x dx dxe Pdx; apply: (fOg (x, dx)); split=> //=.
move: dxe; rewrite gt_max !lt_min => /andP[/andP [dxe11 _] /andP [_ dxe22]].
Expand Down
1 change: 0 additions & 1 deletion reals/all_reals.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,3 @@
From mathcomp Require Export signed.
From mathcomp Require Export itv.
From mathcomp Require Export constructive_ereal.
From mathcomp Require Export reals.
Expand Down
Loading

0 comments on commit 89faa96

Please sign in to comment.