summaryrefslogtreecommitdiff
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.v3
1 files changed, 1 insertions, 2 deletions
diff --git a/test-suite/bugs/closed/4873.v b/test-suite/bugs/closed/4873.v
index f2f917b4..39299883 100644
--- a/test-suite/bugs/closed/4873.v
+++ b/test-suite/bugs/closed/4873.v
@@ -1,6 +1,5 @@
Require Import Coq.Classes.Morphisms.
Require Import Relation_Definitions.
-Require Import Coq.Compat.Coq85.
Fixpoint tuple' T n : Type :=
match n with
@@ -69,4 +68,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.