summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/3453.v
blob: 4ee9b400a327c666fd8eb0a33d10440bf97717e5 (plain)
1
2
3
4
5
6
7
8
9
10
Set Primitive Projections.
Record Foo := { bar : Set }.
Class Baz (F : Foo) := { qux : F.(bar) }.
Coercion qux : Baz >-> bar.

Definition f : Foo := {| bar := nat |}.
Canonical Structure f.
Check (fun b : Baz f => b : _.(bar)).

(* Error: Found target class bar instead of bar. *)