aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Compare.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Arith/Compare.v')
-rwxr-xr-xtheories/Arith/Compare.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/theories/Arith/Compare.v b/theories/Arith/Compare.v
index f98115e6b..5b12033dc 100755
--- a/theories/Arith/Compare.v
+++ b/theories/Arith/Compare.v
@@ -9,6 +9,7 @@
(*i $Id$ i*)
(** Equality is decidable on [nat] *)
+Import nat_scope.
Lemma not_eq_sym : (A:Set)(p,q:A)(~p=q) -> ~(q=p).
Proof sym_not_eq.