aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Minus.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-12 19:20:04 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-12 19:20:04 +0000
commite10135925fa344ead0eb760c2c0fb7167d8dfc74 (patch)
treec00f1058346af155c3f54a297b452a1edd640197 /theories/Arith/Minus.v
parent634d52825790d8818883549616b3c8807655d2b8 (diff)
Independance vis a vis noms variables liees; partie sur bool dans Zbool
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4876 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Minus.v')
-rwxr-xr-xtheories/Arith/Minus.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Arith/Minus.v b/theories/Arith/Minus.v
index c8e9a5d40..658c25194 100755
--- a/theories/Arith/Minus.v
+++ b/theories/Arith/Minus.v
@@ -35,7 +35,7 @@ Qed.
Hints Resolve minus_Sn_m : arith v62.
Theorem pred_of_minus : (x:nat)(pred x)=(minus x (S O)).
-NewInduction x; Simpl; Auto with arith.
+Intro x; NewInduction x; Simpl; Auto with arith.
Qed.
(** Diagonal *)