aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/opened/3459.v
blob: db42d960535e03c05494fa11906e1d5aa6d37311 (plain)
1
2
3
4
5
6
7
8
9
Goal 1 = 2.
Proof.
match goal with
  | [ |- context G[2] ] => let y := constr:(fun x => $(let r := constr:(@eq Set x x) in
                                                       clear x;
                                                       exact r)$) in
                           pose y
end.
Abort.