aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/QArith/Qcabs.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/QArith/Qcabs.v')
-rw-r--r--theories/QArith/Qcabs.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/QArith/Qcabs.v b/theories/QArith/Qcabs.v
index 1883c77be..09908665e 100644
--- a/theories/QArith/Qcabs.v
+++ b/theories/QArith/Qcabs.v
@@ -126,4 +126,4 @@ Proof.
destruct (proj1 (Qcabs_Qcle_condition x 0)) as [A B].
+ rewrite H; apply Qcle_refl.
+ apply Qcle_antisym; auto.
-Qed. \ No newline at end of file
+Qed.