aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/EqNat.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/EqNat.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/EqNat.v')
-rwxr-xr-xtheories/Arith/EqNat.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Arith/EqNat.v b/theories/Arith/EqNat.v
index 9b1bca7c4..a0ba5127d 100755
--- a/theories/Arith/EqNat.v
+++ b/theories/Arith/EqNat.v
@@ -64,7 +64,7 @@ Fixpoint beq_nat [n:nat] : nat -> bool :=
Lemma beq_nat_refl : (x:nat)true=(beq_nat x x).
Proof.
- NewInduction x; Simpl; Auto.
+ Intro x; NewInduction x; Simpl; Auto.
Qed.
Definition beq_nat_eq : (x,y:nat)true=(beq_nat x y)->x=y.