aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/4354.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2015-10-09 15:41:48 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2015-10-09 15:41:48 +0200
commit5e1296a5cae4ae0ab84ddbe7b0ec71959861af97 (patch)
treed69205153e357369fe5ecd674b3a4003a4714c6e /test-suite/bugs/closed/4354.v
parentf3c4dc6fb350b318ccc3af3a0e9aecb977b25744 (diff)
Refine fix for handling of the universe contexts of hints, depending on
their polymorphic status _and_ locality.
Diffstat (limited to 'test-suite/bugs/closed/4354.v')
-rw-r--r--test-suite/bugs/closed/4354.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/test-suite/bugs/closed/4354.v b/test-suite/bugs/closed/4354.v
index 6a2f9672d..e71ddaf71 100644
--- a/test-suite/bugs/closed/4354.v
+++ b/test-suite/bugs/closed/4354.v
@@ -3,8 +3,9 @@ Class Lift (T : Type).
Axiom closed_increment : forall {T} {H : Lift T}, True.
Create HintDb core.
Lemma closed_monotonic T (H : Lift T) : True.
+Proof.
+ Set Printing Universes.
auto using closed_increment. Show Universes.
Qed.
-
(* also fails with -nois, so the content of the hint database does not matter
*) \ No newline at end of file