aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/coqchk
diff options
context:
space:
mode:
authorGravatar Gaëtan Gilbert <gaetan.gilbert@skyskimmer.net>2018-04-20 17:06:20 +0200
committerGravatar Gaëtan Gilbert <gaetan.gilbert@skyskimmer.net>2018-04-20 17:06:20 +0200
commit26da42bee0b32c0f7316475e64ca2204c740efd2 (patch)
tree2f9625fb70a68e33494090d470b11f8a7f3c4089 /test-suite/coqchk
parent9a4ca53a3a021cb16de7706ec79a26e49f54de49 (diff)
Fix #6798: coqchk ignores ugraph when comparing constant instances
Diffstat (limited to 'test-suite/coqchk')
-rw-r--r--test-suite/coqchk/univ.v13
1 files changed, 13 insertions, 0 deletions
diff --git a/test-suite/coqchk/univ.v b/test-suite/coqchk/univ.v
index 19eea94b1..fcd740927 100644
--- a/test-suite/coqchk/univ.v
+++ b/test-suite/coqchk/univ.v
@@ -46,3 +46,16 @@ Inductive constraint4 : (Type -> Type) -> Type
:= mk_constraint4 : let U1 := Type in
let U2 := Type in
constraint4 (fun x : U1 => (x : U2)).
+
+Module CMP_CON.
+ (* Comparison of opaque constants MUST be up to the universe graph.
+ See #6798. *)
+ Universe big.
+
+ Polymorphic Lemma foo@{u} : Type@{big}.
+ Proof. exact Type@{u}. Qed.
+
+ Universes U V.
+
+ Definition yo : foo@{U} = foo@{V} := eq_refl.
+End CMP_CON.