aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-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