aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/1951.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2014-06-23 18:29:07 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2014-06-23 18:31:17 +0200
commit1f11c1f1366b4c82e2e596b3cc97ee0052189741 (patch)
treeda1ad0cc24aea020f386d729b8dc8e0442537931 /test-suite/bugs/closed/1951.v
parentee2adce57aac1ffe21681a9d31a8e8bc4f94210b (diff)
Fix for bug 1951, allowing at least fully-applied inductives types to be used
for building polymorphic instances of template polymorphic inductives.
Diffstat (limited to 'test-suite/bugs/closed/1951.v')
-rw-r--r--test-suite/bugs/closed/1951.v10
1 files changed, 5 insertions, 5 deletions
diff --git a/test-suite/bugs/closed/1951.v b/test-suite/bugs/closed/1951.v
index 12c0ef9bf..7558b0b86 100644
--- a/test-suite/bugs/closed/1951.v
+++ b/test-suite/bugs/closed/1951.v
@@ -5,11 +5,11 @@ Set Printing Universes.
Inductive enc (A:Type (*1*)) (* : Type.1 *) := C : A -> enc A.
-Definition id (X:Type(*5*)) (x:X) := x.
+Definition id (X:Type(*4*)) (x:X) := x.
-Lemma test : let S := Type(*6 : 7*) in enc S -> S.
+Lemma test : let S := Type(*5 : 6*) in enc S -> S.
simpl; intros.
-apply enc.
+refine (enc _).
apply id.
apply Prop.
Defined.
@@ -26,7 +26,7 @@ b : (list a) -> a. (* i don't know if this *)
Inductive sg : Type := Sg. (* single *)
Definition ipl2 (P : a -> Type) := (* in Prop, that means P is true forall *)
-fold_right (fun x => prod (P x)) sg. (* the elements of a given list *)
+ fold_right (fun x => fun A => prod (P x) A) sg. (* the elements of a given list *)
Definition ind
: forall S : a -> Type,
@@ -55,7 +55,7 @@ Defined.
Lemma k' : a -> Type. (* same lemma but with our bug *)
intro;pattern H;apply ind;intros.
- apply prod.
+ refine (prod _ _).
induction ls.
exact sg.
exact sg.