aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/QArith
diff options
context:
space:
mode:
authorGravatar Théo Zimmermann <theo.zimmermann@univ-paris-diderot.fr>2017-03-14 16:22:48 +0100
committerGravatar Théo Zimmermann <theo.zimmermann@univ-paris-diderot.fr>2017-03-14 16:22:48 +0100
commit88c02e02a7b6067c78608e9ea526f81fd122edab (patch)
tree305a35044440f6d338165f4f512f31f115f97556 /theories/QArith
parent43524c6689f372b32770c20d19866f2f4edb4cc6 (diff)
Fix 3 unused-intro-pattern warnings in stdlib.
Diffstat (limited to 'theories/QArith')
-rw-r--r--theories/QArith/Qround.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/QArith/Qround.v b/theories/QArith/Qround.v
index 0ed6d557c..e94ef408d 100644
--- a/theories/QArith/Qround.v
+++ b/theories/QArith/Qround.v
@@ -141,7 +141,7 @@ Qed.
Lemma Zdiv_Qdiv (n m: Z): (n / m)%Z = Qfloor (n / m).
Proof.
unfold Qfloor. intros. simpl.
- destruct m as [?|?|p]; simpl.
+ destruct m as [ | | p]; simpl.
now rewrite Zdiv_0_r, Z.mul_0_r.
now rewrite Z.mul_1_r.
rewrite <- Z.opp_eq_mul_m1.