summaryrefslogtreecommitdiff
path: root/theories/QArith/Qcabs.v
diff options
context:
space:
mode:
authorGravatar Benjamin Barenblat <bbaren@debian.org>2018-12-29 14:31:32 -0500
committerGravatar Benjamin Barenblat <bbaren@debian.org>2018-12-29 14:31:32 -0500
commit2708a015fcf65f72328be4296a00dd32b1f1c17a (patch)
tree696f9b5fb84817e1a5c8d9271976a92e25aef18a /theories/QArith/Qcabs.v
parentd7d80c5bea564b7cb0eadc33e9ee38c9d9de1cd8 (diff)
parent9043add656177eeac1491a73d2f3ab92bec0013c (diff)
Updated version 8.8.2 from 'upstream/8.8.2'
Diffstat (limited to 'theories/QArith/Qcabs.v')
-rw-r--r--theories/QArith/Qcabs.v14
1 files changed, 8 insertions, 6 deletions
diff --git a/theories/QArith/Qcabs.v b/theories/QArith/Qcabs.v
index c0ababff..f45868a7 100644
--- a/theories/QArith/Qcabs.v
+++ b/theories/QArith/Qcabs.v
@@ -1,9 +1,11 @@
(************************************************************************)
-(* v * The Coq Proof Assistant / The Coq Development Team *)
-(* <O___,, * INRIA - CNRS - LIX - LRI - PPS - Copyright 1999-2016 *)
+(* * The Coq Proof Assistant / The Coq Development Team *)
+(* v * INRIA, CNRS and contributors - Copyright 1999-2018 *)
+(* <O___,, * (see CREDITS file for the list of authors) *)
(* \VV/ **************************************************************)
-(* // * This file is distributed under the terms of the *)
-(* * GNU Lesser General Public License Version 2.1 *)
+(* // * This file is distributed under the terms of the *)
+(* * GNU Lesser General Public License Version 2.1 *)
+(* * (see LICENSE file for the text of the license) *)
(************************************************************************)
(** * An absolute value for normalized rational numbers. *)
@@ -22,7 +24,7 @@ Lemma Qcabs_canon (x : Q) : Qred x = x -> Qred (Qabs x) = Qabs x.
Proof. intros H; now rewrite (Qred_abs x), H. Qed.
Definition Qcabs (x:Qc) : Qc := {| canon := Qcabs_canon x (canon x) |}.
-Notation "[ q ]" := (Qcabs q) (q at next level, format "[ q ]") : Qc_scope.
+Notation "[ q ]" := (Qcabs q) : Qc_scope.
Ltac Qc_unfolds :=
unfold Qcabs, Qcminus, Qcopp, Qcplus, Qcmult, Qcle, Q2Qc, this.
@@ -126,4 +128,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.