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

Require Import Setoid.

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