Skip to content

Commit

Permalink
adapt to coq/coq#19801 (deprecation of ZArith_base, Zeq_bool)
Browse files Browse the repository at this point in the history
  • Loading branch information
andres-erbsen committed Nov 3, 2024
1 parent 1f014ff commit b08fd06
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 2 deletions.
4 changes: 3 additions & 1 deletion BigQ/QMake.v
Original file line number Diff line number Diff line change
Expand Up @@ -181,7 +181,9 @@ Module Make (NN:NType)(ZZ:ZType)(Import NZ:NType_ZType NN ZZ) <: QType.

Theorem spec_eq_bool: forall x y, eq_bool x y = Qeq_bool [x] [y].
Proof.
intros. unfold eq_bool. rewrite spec_compare. reflexivity.
unfold eq_bool; intros.
apply eq_true_iff_eq; rewrite Qeq_bool_iff, spec_compare, Qeq_alt.
case Qcompare; intuition congruence.
Qed.

(** [check_int] : is a reduced fraction [n/d] in fact a integer ? *)
Expand Down
2 changes: 1 addition & 1 deletion BigZ/BigZ.v
Original file line number Diff line number Diff line change
Expand Up @@ -10,7 +10,7 @@

Require Export BigN.
Require Import ZProperties ZDivFloor ZSig ZSigZAxioms ZMake Ring Lia.
Import Zpow_def Zdiv.
Import BinNat Zpow_def Zdiv.

(** * [BigZ] : arbitrary large efficient integers.
Expand Down

0 comments on commit b08fd06

Please sign in to comment.