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

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