summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/shouldfail/2586.v
blob: 6111a6415f1cffdf4e31647fe347c01904d2806a (plain)
1
2
3
4
5
Require Import Setoid SetoidClass Program.

Goal forall `(Setoid nat) x y, x == y -> S x == S y.
  intros.
  clsubst H0.