aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3590.v
blob: 3440f0e8063078a2d16991a2c54a3faa9d0a4cde (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
Require Import TestSuite.admit.
(* Set Primitive Projections. *)
Set Implicit Arguments.
Record prod A B := pair { fst : A ; snd : B }.
Definition idS := Set.
Goal forall x y : prod Set Set, fst x = fst y.
  intros.
  change (@fst _ _ ?z) with (@fst Set idS z) at 2.
  Unshelve.
  admit.
Qed.
  
(* Toplevel input, characters 20-58:
Error: Failed to get enough information from the left-hand side to type the
right-hand side. *)