aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/4544.v
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-05-03 15:06:11 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-05-03 16:05:08 +0200
commitb6e796a8ef956fa25bfeba84545f25b2cfb3aaf9 (patch)
treeda87235dd73f6425ea980100894ccc910a0ec877 /test-suite/bugs/closed/4544.v
parent00a13c3c014e2729d17ad8e8191f20586ae3b52b (diff)
Fix bug #3825: Universe annotations on notations should pass through or be rejected.
Diffstat (limited to 'test-suite/bugs/closed/4544.v')
-rw-r--r--test-suite/bugs/closed/4544.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/bugs/closed/4544.v b/test-suite/bugs/closed/4544.v
index d14cc86fc..048f31ce3 100644
--- a/test-suite/bugs/closed/4544.v
+++ b/test-suite/bugs/closed/4544.v
@@ -841,7 +841,7 @@ End Truncation_Modalities.
Module Import TrM := Modalities_Theory Truncation_Modalities.
-Definition merely (A : Type@{i}) : hProp@{i} := BuildhProp (Trunc -1 A).
+Definition merely (A : Type@{i}) : hProp := BuildhProp (Trunc -1 A).
Notation IsSurjection := (IsConnMap -1).