Skip to content

Commit

Permalink
Merge pull request #94 from andres-erbsen/less-ZArith_base
Browse files Browse the repository at this point in the history
adapt to coq/coq#19801 (replacing ZArith_base, Zeq_bool)
  • Loading branch information
proux01 authored Jan 7, 2025
2 parents 97da402 + 0b1a1b2 commit cc2d9ee
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 @@ -11,7 +11,7 @@
From Stdlib Require Import ZProperties ZDivFloor Ring Lia.
Require Export BigN.
Require Import ZSig ZSigZAxioms ZMake.
Import Zpow_def Zdiv.
Import BinNat Zpow_def Zdiv.

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

0 comments on commit cc2d9ee

Please sign in to comment.