aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3978.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-02-12 22:59:41 +0100
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-02-12 22:59:41 +0100
commit1e1a2f1803c57cc1697e294a7610b76a95661687 (patch)
treecc683aa3b940c36ab3f5c692693bfeeb257855d4 /test-suite/bugs/closed/3978.v
parent8c5bfa0f00b80979473bba26c1b9a1410667e032 (diff)
COMPATIBILITY: add note about the change of behavior of Instance foo :=
{| |}. Add test-suite files for closed bugs.
Diffstat (limited to 'test-suite/bugs/closed/3978.v')
-rw-r--r--test-suite/bugs/closed/3978.v27
1 files changed, 27 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3978.v b/test-suite/bugs/closed/3978.v
new file mode 100644
index 000000000..26e021e71
--- /dev/null
+++ b/test-suite/bugs/closed/3978.v
@@ -0,0 +1,27 @@
+Require Import Structures.OrderedType.
+Require Import Structures.OrderedTypeEx.
+
+Module Type M. Parameter X : Type.
+
+Declare Module Export XOrd : OrderedType
+ with Definition t := X
+ with Definition eq := @Logic.eq X.
+End M.
+
+Module M' : M.
+ Definition X := nat.
+
+ Module XOrd := Nat_as_OT.
+End M'.
+
+Module Type MyOt.
+ Parameter t : Type.
+ Parameter eq : t -> t -> Prop.
+End MyOt.
+
+Module Type M2. Parameter X : Type.
+
+Declare Module Export XOrd : MyOt
+ with Definition t := X
+ with Definition eq := @Logic.eq X.
+End M2.