summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/1915.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/bugs/closed/1915.v')
-rw-r--r--test-suite/bugs/closed/1915.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/bugs/closed/1915.v b/test-suite/bugs/closed/1915.v
index 7e62437d..2b0aed8c 100644
--- a/test-suite/bugs/closed/1915.v
+++ b/test-suite/bugs/closed/1915.v
@@ -3,4 +3,4 @@ Require Import Setoid.
Fail Goal forall x, impl True (x = 0) -> x = 0 -> False.
(*intros x H E.
-rewrite H in E.*) \ No newline at end of file
+rewrite H in E.*)