aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar werner <werner@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-06-12 16:03:32 +0000
committerGravatar werner <werner@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-06-12 16:03:32 +0000
commit471e50d415a30191f0ebdaa707ce1889990d4923 (patch)
tree475807f0d3c718c6f43fbd8dee883da274daf142 /theories
parent7db3c187811a21761c7d13f4b5de8562eb59b5a9 (diff)
Changing the definitions of pred and minus in the style of GG
in order for them to preserve the structural order. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11115 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rw-r--r--theories/Init/Peano.v6
1 files changed, 5 insertions, 1 deletions
diff --git a/theories/Init/Peano.v b/theories/Init/Peano.v
index a7e1a39aa..27a8c5a91 100644
--- a/theories/Init/Peano.v
+++ b/theories/Init/Peano.v
@@ -164,7 +164,11 @@ Notation mult_succ_r_reverse := mult_n_Sm (only parsing).
Fixpoint minus (n m:nat) {struct n} : nat :=
match n, m with
| O, _ => n
- | S k, O => S k
+ | S k, O => n
+(*=======
+
+ | O, _ => n
+ | S k, O => S k *)
| S k, S l => k - l
end