aboutsummaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/bug_3633.v
blob: 7a82a2685e0ff61be604fa93398ea3ae63a56292 (plain)
1
2
3
4
5
6
7
8
9
10
Set Typeclasses Strict Resolution.
Class Contr (A : Type) := { center : A }.
Definition foo {A} `{Contr A} : A.
Proof.
  apply center.
  Undo.
  (* Ensure the constraints are solved independently, otherwise a frozen ?A
  makes a search for Contr ?A fail when finishing to apply (fun x => x) *)
  apply (fun x => x), center.
Qed.