summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/shouldsucceed/1483.v
blob: a3d7f168308abfeafd294ace152ecef75ac7f12c (plain)
1
2
3
4
5
6
7
8
9
10
Require Import BinPos.

Definition P := (fun x : positive => x = xH).

Goal forall (p q : positive), P q -> q = p -> P p.
intros; congruence.
Qed.