aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Sets/Integers.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Sets/Integers.v')
-rw-r--r--theories/Sets/Integers.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/theories/Sets/Integers.v b/theories/Sets/Integers.v
index 01d3bda37..15c1b665e 100644
--- a/theories/Sets/Integers.v
+++ b/theories/Sets/Integers.v
@@ -79,6 +79,7 @@ Section Integers_sect.
auto with sets arith.
apply Inhabited_intro with (x := 0).
apply Integers_defn.
+ exact le_Order.
Defined.
Lemma le_total_order : Totally_ordered nat nat_po Integers.