aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
authorMatthieu Sozeau2019-08-26 16:10:41 +0200
committerMatthieu Sozeau2019-08-26 16:21:46 +0200
commit09bf7631fa92a2f6d93e940b8730a2a053ba4efc (patch)
tree1296867e04a171bbf842a39955ec5536129c6f58
parent1e434fe4421bee0b1928fd015fb60025ec6c2833 (diff)
Test-suite fixes from Hugo
-rw-r--r--test-suite/success/Template.v19
1 files changed, 18 insertions, 1 deletions
diff --git a/test-suite/success/Template.v b/test-suite/success/Template.v
index c38b761f1f..656362b8fc 100644
--- a/test-suite/success/Template.v
+++ b/test-suite/success/Template.v
@@ -59,7 +59,7 @@ Module ExplicitTemplate.
#[universes(template)]
Inductive identity@{i} (A : Type@{i}) (a : A) : A -> Type@{i} := id_refl : identity A a a.
- (* Weird intraction of template polymorphism and inductives
+ (* Weird interaction of template polymorphism and inductive types
which naturally fall in Prop: this one is template polymorphic but not on i:
it just lives in any universe *)
Check (identity Type nat nat : Prop).
@@ -155,3 +155,20 @@ Module TestTemplateAttribute.
End Foo.
End TestTemplateAttribute.
+
+Module SharingWithoutSection.
+Inductive Foo A (S:= fun _ => Set : ltac:(let ty := type of A in exact ty))
+ := foo : S A -> Foo A.
+Fail Check Foo True : Prop.
+End SharingWithoutSection.
+
+Module OkNotCovered.
+(* Here it happens that box is safe but we don't see it *)
+Section S.
+Universe u.
+Variable A : Type@{u}.
+Inductive box (A:Type@{u}) := Box : A -> box A.
+Definition B := Set : Type@{u}.
+End S.
+Fail Check box True : Prop.
+End OkNotCovered.