summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/1900.v
blob: 6eea5db0832c52bb84aede91f13ed5e796bd719c (plain)
1
2
3
4
5
6
7
8
Parameter A : Type .

Definition eq_A := @eq A.

Goal forall x, eq_A x x.
intros.
reflexivity.
Qed.