summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/1915.v
blob: 7e62437d7b1afa8ac5bf5838e698bb17ff81d96c (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.*)