aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Peano_dec.v
diff options
context:
space:
mode:
authorGravatar mohring <mohring@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-19 12:25:05 +0000
committerGravatar mohring <mohring@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-19 12:25:05 +0000
commitbdbbb1bea47909ad5d0daffd77e090ef9b59d826 (patch)
tree4d1265dfb29299fb395a554a3b32eb550b4662a2 /theories/Arith/Peano_dec.v
parent45aa164112c77d61f726d5db32041c9518ed378a (diff)
Mise de (*i autour CVS info
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1619 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Peano_dec.v')
-rwxr-xr-xtheories/Arith/Peano_dec.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Arith/Peano_dec.v b/theories/Arith/Peano_dec.v
index 5ee33d156..b02d5a324 100755
--- a/theories/Arith/Peano_dec.v
+++ b/theories/Arith/Peano_dec.v
@@ -6,9 +6,9 @@
(* * GNU Lesser General Public License Version 2.1 *)
(***********************************************************************)
-Require Decidable.
-(* $Id$ *)
+(*i $Id$ i*)
+Require Decidable.
Theorem O_or_S : (n:nat)({m:nat|(S m)=n})+{O=n}.
Proof.