Skip to content

Commit cc2d9ee

Browse files
authored
Merge pull request #94 from andres-erbsen/less-ZArith_base
adapt to rocq-prover/rocq#19801 (replacing ZArith_base, Zeq_bool)
2 parents 97da402 + 0b1a1b2 commit cc2d9ee

File tree

2 files changed

+4
-2
lines changed

2 files changed

+4
-2
lines changed

BigQ/QMake.v

Lines changed: 3 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -181,7 +181,9 @@ Module Make (NN:NType)(ZZ:ZType)(Import NZ:NType_ZType NN ZZ) <: QType.
181181

182182
Theorem spec_eq_bool: forall x y, eq_bool x y = Qeq_bool [x] [y].
183183
Proof.
184-
intros. unfold eq_bool. rewrite spec_compare. reflexivity.
184+
unfold eq_bool; intros.
185+
apply eq_true_iff_eq; rewrite Qeq_bool_iff, spec_compare, Qeq_alt.
186+
case Qcompare; intuition congruence.
185187
Qed.
186188

187189
(** [check_int] : is a reduced fraction [n/d] in fact a integer ? *)

BigZ/BigZ.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -11,7 +11,7 @@
1111
From Stdlib Require Import ZProperties ZDivFloor Ring Lia.
1212
Require Export BigN.
1313
Require Import ZSig ZSigZAxioms ZMake.
14-
Import Zpow_def Zdiv.
14+
Import BinNat Zpow_def Zdiv.
1515

1616
(** * [BigZ] : arbitrary large efficient integers.
1717

0 commit comments

Comments
 (0)