From 26da42bee0b32c0f7316475e64ca2204c740efd2 Mon Sep 17 00:00:00 2001 From: Gaƫtan Gilbert Date: Fri, 20 Apr 2018 17:06:20 +0200 Subject: Fix #6798: coqchk ignores ugraph when comparing constant instances --- test-suite/coqchk/univ.v | 13 +++++++++++++ 1 file changed, 13 insertions(+) (limited to 'test-suite/coqchk') 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. -- cgit v1.2.3