aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/Cases.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-12-18 07:00:50 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-12-18 07:00:50 +0000
commit7f4b6b875daaf1d31ff74a58d8916c2a4889cf3a (patch)
tree4c932205d7eb8ad6306ac1d708ee64874856f8d1 /test-suite/success/Cases.v
parent693b8a7a4dc4535d2aa2912deec2cb21deb39c75 (diff)
Taking into account the possibility of having a type of type which is
an evar in typing.ml. Thanks to HoTT people for noticing the problem. Fixed behavior of e_typing git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16092 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/Cases.v')
-rw-r--r--test-suite/success/Cases.v6
1 files changed, 6 insertions, 0 deletions
diff --git a/test-suite/success/Cases.v b/test-suite/success/Cases.v
index f445ca8ea..c9a3c08ef 100644
--- a/test-suite/success/Cases.v
+++ b/test-suite/success/Cases.v
@@ -1865,3 +1865,9 @@ Type (fun n => match n with
| Z0 => true
| _ => false
end).
+
+(* Check that types with unknown sort, as A below, are not fatal to
+ the pattern-matching compilation *)
+
+Definition transport {A} (P : A->Type) {x y : A} (p : x=y) (u : P x) : P y :=
+ match p with eq_refl => u end.