From 20adaabfa96744442f201287e2900b1575614577 Mon Sep 17 00:00:00 2001 From: Pierre Letouzey Date: Fri, 26 Feb 2016 20:01:18 +0100 Subject: Qcanon : fix names of lemmas Qcle_alt & Qcge_alt (were Qle_alt & Qge_alt) --- theories/QArith/Qcanon.v | 4 ++-- 1 file changed, 2 insertions(+), 2 deletions(-) (limited to 'theories/QArith') diff --git a/theories/QArith/Qcanon.v b/theories/QArith/Qcanon.v index 86be28d7b..078926e32 100644 --- a/theories/QArith/Qcanon.v +++ b/theories/QArith/Qcanon.v @@ -130,12 +130,12 @@ Proof. intros; exact (Qgt_alt p q). Qed. -Lemma Qle_alt : forall p q, (p<=q) <-> (p?=q <> Gt). +Lemma Qcle_alt : forall p q, (p<=q) <-> (p?=q <> Gt). Proof. intros; exact (Qle_alt p q). Qed. -Lemma Qge_alt : forall p q, (p>=q) <-> (p?=q <> Lt). +Lemma Qcge_alt : forall p q, (p>=q) <-> (p?=q <> Lt). Proof. intros; exact (Qge_alt p q). Qed. -- cgit v1.2.3