summaryrefslogtreecommitdiff
path: root/test-suite/failure/guard-cofix.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/failure/guard-cofix.v')
-rw-r--r--test-suite/failure/guard-cofix.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/failure/guard-cofix.v b/test-suite/failure/guard-cofix.v
index eda4a186..3ae87705 100644
--- a/test-suite/failure/guard-cofix.v
+++ b/test-suite/failure/guard-cofix.v
@@ -40,4 +40,4 @@ Fail CoFixpoint loop' : CoFalse :=
Omega match eq_sym H in _ = T return T with eq_refl => loop' end
end.
-Fail Definition ff' : False := match loop' with CF _ t => t end. \ No newline at end of file
+Fail Definition ff' : False := match loop' with CF _ t => t end.