aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/4873.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/bugs/closed/4873.v')
-rw-r--r--test-suite/bugs/closed/4873.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/bugs/closed/4873.v b/test-suite/bugs/closed/4873.v
index f2f917b4e..3be36d847 100644
--- a/test-suite/bugs/closed/4873.v
+++ b/test-suite/bugs/closed/4873.v
@@ -69,4 +69,4 @@ Proof.
destruct xs; simpl; intros; subst; auto.
generalize dependent t. simpl in *.
induction xs; simpl in *; intros; congruence.
-Qed. \ No newline at end of file
+Qed.