summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/1915.v
blob: 2b0aed8c7d6f5909bfcd05623c6a16a1302936ac (plain)
1
2
3
4
5
6

Require Import Setoid.

Fail Goal forall x, impl True (x = 0) -> x = 0 -> False.
(*intros x H E.
rewrite H in E.*)