summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/3633.v
blob: 52bb307271af4cc161bd0f04919c7e2a03a5cd12 (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.