Skip to content

Commit

Permalink
Merge pull request #132 from andres-erbsen/less-ZArith_base
Browse files Browse the repository at this point in the history
fully qualify unimported ZArith lemmas (for coq/coq#19801)
  • Loading branch information
spitters authored Nov 3, 2024
2 parents 5faa2f7 + ef36545 commit 9db3142
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 2 deletions.
2 changes: 1 addition & 1 deletion implementations/QType_rationals.v
Original file line number Diff line number Diff line change
Expand Up @@ -159,7 +159,7 @@ Qed.
Next Obligation.
rewrite spec_compare in *.
destruct (Qcompare_spec (to_Q x) (to_Q y)); try discriminate; try intuition.
now apply Zeq_le.
now apply Zorder.Zeq_le.
now apply orders.lt_le.
Qed.

Expand Down
2 changes: 1 addition & 1 deletion implementations/fast_rationals.v
Original file line number Diff line number Diff line change
Expand Up @@ -58,7 +58,7 @@ Proof.
case_eq (BigN.eqb d BigN.zero); intros Ed2; [reflexivity |].
rewrite BigZ.spec_compare in Ed.
destruct (proj2 (not_true_iff_false _) Ed2).
apply BigN.eqb_eq. symmetry. now apply Zcompare_Eq_eq.
apply BigN.eqb_eq. symmetry. now apply Zcompare.Zcompare_Eq_eq.
unfold BigQ.mul. simpl. rewrite right_identity. reflexivity.
destruct (BigZ.compare_spec BigZ.zero (BigZ.Pos d)); try discriminate.
destruct (orders.lt_not_le_flip 0 ('d : bigZ)); trivial.
Expand Down

0 comments on commit 9db3142

Please sign in to comment.