aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/autointros.v
diff options
context:
space:
mode:
authorGravatar serpyc <serpyc@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-10-04 10:40:03 +0000
committerGravatar serpyc <serpyc@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-10-04 10:40:03 +0000
commit88909c92cad0044dac83539b2b3d385242ed851e (patch)
treef8c946fc168920aab8c7e47cf875be8404f1bd10 /test-suite/success/autointros.v
parent4b993912cc6c6135e41ea959f934fa73d1da05ab (diff)
Removal of trailing spaces.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12371 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/autointros.v')
-rw-r--r--test-suite/success/autointros.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/test-suite/success/autointros.v b/test-suite/success/autointros.v
index 71054e141..0a0812711 100644
--- a/test-suite/success/autointros.v
+++ b/test-suite/success/autointros.v
@@ -9,7 +9,7 @@ with odd : nat -> Prop :=
Lemma foo {n : nat} (E : even n) : even (S (S n))
with bar {n : nat} (O : odd n) : odd (S (S n)).
-Proof. destruct E. constructor. constructor. apply even_odd. apply (bar _ H).
- destruct O. repeat constructor. apply odd_even. apply (foo _ H).
+Proof. destruct E. constructor. constructor. apply even_odd. apply (bar _ H).
+ destruct O. repeat constructor. apply odd_even. apply (foo _ H).
Defined.