Skip to content

Commit

Permalink
Treat a deprecation warning about Qint
Browse files Browse the repository at this point in the history
  • Loading branch information
pi8027 committed Jul 2, 2024
1 parent 027788b commit c9597ff
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 8 deletions.
8 changes: 2 additions & 6 deletions meta.yml
Original file line number Diff line number Diff line change
Expand Up @@ -38,10 +38,6 @@ supported_coq_versions:
opam: '{(>= "8.16" & < "8.20~") | (= "dev")}'

tested_coq_opam_versions:
- version: '2.0.0-coq-8.16'
repo: 'mathcomp/mathcomp'
- version: '2.0.0-coq-8.18'
repo: 'mathcomp/mathcomp'
- version: '2.1.0-coq-8.16'
repo: 'mathcomp/mathcomp'
- version: '2.1.0-coq-8.18'
Expand All @@ -64,9 +60,9 @@ ci_cron_schedule: '0 5 * * *'
dependencies:
- opam:
name: coq-mathcomp-ssreflect
version: '{(>= "2.0.0" & < "2.3~") | (= "dev")}'
version: '{(>= "2.1.0" & < "2.3~") | (= "dev")}'
description: |-
[MathComp ssreflect 2.0 or later](https://math-comp.github.io)
[MathComp ssreflect 2.1 or later](https://math-comp.github.io)
- opam:
name: coq-mathcomp-algebra
description: |-
Expand Down
4 changes: 2 additions & 2 deletions theories/realprop.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
(* (c) Copyright 2006-2018 Microsoft Corporation and Inria. *)
(* Distributed under the terms of CeCILL-B. *)
From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssrnat div order.
From mathcomp Require Import ssralg ssrnum ssrint rat intdiv.
From mathcomp Require Import ssralg ssrnum ssrint archimedean rat intdiv.

Check failure on line 4 in theories/realprop.v

View workflow job for this annotation

GitHub Actions / build (mathcomp/mathcomp:2.0.0-coq-8.18)

Cannot find a physical path bound to logical path

Check failure on line 4 in theories/realprop.v

View workflow job for this annotation

GitHub Actions / build (mathcomp/mathcomp:2.0.0-coq-8.16)

Cannot find a physical path bound to logical path
From Coq Require Import Morphisms Setoid.
From fourcolor Require Import real realsyntax.

Expand Down Expand Up @@ -46,7 +46,7 @@ Definition max x y : R := IF x >= y then x else y.
Definition intR m : R := match m with Posz n => n%:R | Negz n => - n.+1%:R end.

Definition ratR (a : rat) :=
if a \is a Qint then intR (numq a) else intR (numq a) / intR (denq a).
if a \is a Num.int then intR (numq a) else intR (numq a) / intR (denq a).

Inductive floor_set x : Real.set R :=
FloorSet m of intR m <= x : floor_set x (intR m).
Expand Down

0 comments on commit c9597ff

Please sign in to comment.