aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_3542.v
blob: e9a846062286a547efe02333a5214bfa06ec9edd (plain)
1
2
3
4
5
6
7
8
Section foo.
  Context {A:Type} {B : A -> Type}.
  Context (f : forall x, B x).
  Goal True.
    pose (r := fun k => existT (fun g => forall x, f x = g x)
                               (fun x => projT1 (k x)) (fun x => projT2 (k x))).
  Abort.
End foo.