aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/EqNat.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Arith/EqNat.v')
-rwxr-xr-xtheories/Arith/EqNat.v3
1 files changed, 3 insertions, 0 deletions
diff --git a/theories/Arith/EqNat.v b/theories/Arith/EqNat.v
index 88cca274b..c42deebd2 100755
--- a/theories/Arith/EqNat.v
+++ b/theories/Arith/EqNat.v
@@ -9,8 +9,11 @@
(*i $Id$ i*)
(** Equality on natural numbers *)
+
Import nat_scope.
+Implicit Variables Type m,n,x,y:nat.
+
Fixpoint eq_nat [n:nat] : nat -> Prop :=
[m:nat]Cases n m of
O O => True