summaryrefslogtreecommitdiff
path: root/test-suite/bugs/opened/4813.v
blob: 2ac55359346a62c174f7ed6df35cf020ee9ed98d (plain)
1
2
3
4
5
Require Import Program.Tactics.

Record T := BT { t : Set }.
Record U (x : T) := BU { u : t x -> Prop }.
Program Definition A (H : unit -> Prop) : U (BT unit) := BU _ H.