From f1a561d847e207433a0ec3e6333798dfa19e4a0c Mon Sep 17 00:00:00 2001 From: Hugo Herbelin Date: Sat, 17 Sep 2016 20:24:36 +0200 Subject: Further "decide equality" tests on demand of Jason. --- theories/Structures/OrdersFacts.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'theories/Structures') diff --git a/theories/Structures/OrdersFacts.v b/theories/Structures/OrdersFacts.v index b059173cb..6f8fc1b32 100644 --- a/theories/Structures/OrdersFacts.v +++ b/theories/Structures/OrdersFacts.v @@ -448,7 +448,7 @@ Lemma leb_compare x y : (x <=? y) = match compare x y with Gt => false | _ => true end. Proof. apply eq_true_iff_eq. rewrite leb_le, <- compare_le_iff. -now destruct compare; split. +now destruct compare. Qed. End BoolOrderFacts. -- cgit v1.2.3