File: bug_16482.v

package info (click to toggle)
coq 9.1.0%2Bdfsg-3
  • links: PTS, VCS
  • area: main
  • in suites: experimental
  • size: 35,964 kB
  • sloc: ml: 239,908; sh: 4,355; python: 2,985; ansic: 2,644; makefile: 874; lisp: 171; javascript: 63; xml: 24; sed: 2
file content (23 lines) | stat: -rw-r--r-- 591 bytes parent folder | download | duplicates (3)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
Set Definitional UIP.
Set Universe Polymorphism.
Set Polymorphic Inductive Cumulativity.

Inductive eqn {A : Type} (x : A) : A -> SProp := refl : @eqn A x x.

Definition Rw {A B : Type} (e : eqn A B) (x : A) : B := match e with | refl _ => x end.

Definition F (A : Type) (P : A -> Type) (Q1 : forall x, P x): SProp.
Proof.
refine (eqn Q1 _).
intro a.
refine (Rw _ (Q1 a)).
reflexivity.
Defined.

Record BTy : Type := {
  typL : Type;
  typP : typL -> Type;
  typQ : forall x, typP x;
  eps : @F typL typP typQ;
}.
(* Anomaly "Uncaught exception Invalid_argument("index out of bounds")." *)