aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-03-19 11:21:13 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2005-03-19 11:21:13 +0000
commite4e5a50f36fee99aef3df84606acfc4563a43124 (patch)
treede14899a224bd2992ffd08d3b5f0518957357376 /test-suite/success
parent868a2e4a7f7461f27f89b35751d29b2fbd409c1a (diff)
Ajout test bug #935
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@6859 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success')
-rw-r--r--test-suite/success/univers.v19
1 files changed, 19 insertions, 0 deletions
diff --git a/test-suite/success/univers.v b/test-suite/success/univers.v
index 8c6f31b4c..a2a1d0dd6 100644
--- a/test-suite/success/univers.v
+++ b/test-suite/success/univers.v
@@ -36,3 +36,22 @@ Proof.
Unfold transitive.
Intros X f g h H1 H2.
Inversion H1.
+Abort.
+
+
+(* Submitted by Bas Spitters (bug report #935) *)
+
+(* This is a problem with the status of the type in LetIn: is it a
+ user-provided one or an inferred one? At the current time, the
+ kernel type-check the type in LetIn, which means that it must be
+ considered as user-provided when calling the kernel. However, in
+ practice it is inferred so that a universe refresh is needed to set
+ its status as "user-provided".
+
+ Especially, universe refreshing was not done for "set/pose" *)
+
+Lemma ind_unsec:(Q:nat->Type)True.
+Intro.
+Pose C:= (m:?)(Q m)->(Q m).
+Exact I.
+Qed.