aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Arith')
-rw-r--r--theories/Arith/Div2.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Arith/Div2.v b/theories/Arith/Div2.v
index 8cef48b69..a9d77c90d 100644
--- a/theories/Arith/Div2.v
+++ b/theories/Arith/Div2.v
@@ -110,7 +110,7 @@ Proof.
split; split; auto with arith. inversion_clear 1. inversion H0.
- (* n = (S (S n')) *)
destruct (even_odd_double n) as ((Ev,Ev'),(Od,Od')).
- split; split; simpl; rewrite ?double_S.
+ split; split; simpl div2; rewrite ?double_S.
+ inversion_clear 1. inversion_clear H0. auto.
+ injection 1. auto with arith.
+ inversion_clear 1. inversion_clear H0. auto.