aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Mult.v
diff options
context:
space:
mode:
authorGravatar notin <notin@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-10-30 09:30:05 +0000
committerGravatar notin <notin@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-10-30 09:30:05 +0000
commita1c45541882eaf4b36459662dcc46810c807a756 (patch)
tree7d593138c8a85d3fd66d9af8d488a99032f96a35 /theories/Arith/Mult.v
parent67040519baa5b82495135a84ae1a79e45a1af42b (diff)
Changement esthétique de la preuve de mult_is_one
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10274 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Mult.v')
-rw-r--r--theories/Arith/Mult.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Arith/Mult.v b/theories/Arith/Mult.v
index 386800934..3c3f3a093 100644
--- a/theories/Arith/Mult.v
+++ b/theories/Arith/Mult.v
@@ -118,7 +118,7 @@ Qed.
Lemma mult_is_one : forall n m, n * m = 1 -> n = 1 /\ m = 1.
Proof.
- induction n as [|n IH].
+ destruct n as [|n].
simpl; intros m H; elim (O_S _ H).
simpl; intros m H.