aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Compat/Coq85.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Compat/Coq85.v')
-rw-r--r--theories/Compat/Coq85.v18
1 files changed, 0 insertions, 18 deletions
diff --git a/theories/Compat/Coq85.v b/theories/Compat/Coq85.v
index 54aeeaa11..490e95c91 100644
--- a/theories/Compat/Coq85.v
+++ b/theories/Compat/Coq85.v
@@ -22,21 +22,3 @@ Global Unset Structural Injection.
Global Unset Shrink Abstract.
Global Unset Shrink Obligations.
Global Set Refolding Reduction.
-
-(** In Coq 8.5, [] meant Vector, and [ ] meant list. Restore this
- behavior, to allow user-defined [] to not override vector
- notations. See https://coq.inria.fr/bugs/show_bug.cgi?id=4785. *)
-
-Require Coq.Lists.List.
-Require Coq.Vectors.VectorDef.
-Module Export Coq.
-Module Export Vectors.
-Module VectorDef.
-Export Coq.Vectors.VectorDef.
-Module VectorNotations.
-Export Coq.Vectors.VectorDef.VectorNotations.
-Notation "[]" := (VectorDef.nil _) : vector_scope.
-End VectorNotations.
-End VectorDef.
-End Vectors.
-End Coq.