aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/opened/HoTT_coq_104.v
blob: ff2da3948ef9fdcf7f59fdaa730102eaf0cd14b2 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
Set Implicit Arguments.

Require Import Logic.

Global Set Universe Polymorphism.
Global Set Asymmetric Patterns.
Local Set Record Elimination Schemes.
Local Set Primitive Projections.

Record prod (A B : Type) : Type :=
  pair { fst : A; snd : B }.

Fail Check fun x : prod Set Set => eq_refl : x = pair (fst x) (snd x).