aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--test-suite/Makefile2
-rw-r--r--test-suite/ide/undo001.fake2
-rw-r--r--test-suite/ide/undo002.fake2
-rw-r--r--test-suite/ide/undo007.fake2
-rw-r--r--test-suite/ide/undo008.fake2
-rw-r--r--test-suite/ide/undo013.fake2
-rw-r--r--test-suite/ide/undo014.fake2
-rw-r--r--test-suite/ide/undo015.fake2
-rw-r--r--test-suite/ide/undo016.fake2
-rw-r--r--test-suite/ide/undo017.fake2
-rw-r--r--test-suite/ide/undo018.fake2
11 files changed, 11 insertions, 11 deletions
diff --git a/test-suite/Makefile b/test-suite/Makefile
index a77b9fffd..e628614ab 100644
--- a/test-suite/Makefile
+++ b/test-suite/Makefile
@@ -94,7 +94,7 @@ clean:
rm -f trace lia.cache
$(SHOW) "RM <**/*.stamp> <**/*.vo> <**/*.log>"
$(HIDE)find . \( \
- -name '*.stamp' -o -name '*.vo' -o -name '*.v.log' \
+ -name '*.stamp' -o -name '*.vo' -o -name '*.log' \
\) -print0 | xargs -0 rm -f
distclean: clean
diff --git a/test-suite/ide/undo001.fake b/test-suite/ide/undo001.fake
index 9e54f4f08..bbaea7e7e 100644
--- a/test-suite/ide/undo001.fake
+++ b/test-suite/ide/undo001.fake
@@ -7,4 +7,4 @@ INTERP Definition foo := 0.
INTERP Definition bar := 1.
REWIND 1
INTERPRAW Check foo.
-INTERPRAW Fail Check bar. \ No newline at end of file
+INTERPRAW Fail Check bar.
diff --git a/test-suite/ide/undo002.fake b/test-suite/ide/undo002.fake
index 36a0e8982..b855b6ea7 100644
--- a/test-suite/ide/undo002.fake
+++ b/test-suite/ide/undo002.fake
@@ -7,4 +7,4 @@ INTERP Definition foo := 0.
INTERP Definition bar := 1.
REWIND 2
INTERPRAW Fail Check foo.
-INTERPRAW Fail Check bar. \ No newline at end of file
+INTERPRAW Fail Check bar.
diff --git a/test-suite/ide/undo007.fake b/test-suite/ide/undo007.fake
index 3b2ca2b6b..87c06dbb3 100644
--- a/test-suite/ide/undo007.fake
+++ b/test-suite/ide/undo007.fake
@@ -14,4 +14,4 @@ INTERP Definition f := O.
INTERP assert True by trivial.
INTERP trivial.
INTERP Qed.
-INTERPRAW Check e. \ No newline at end of file
+INTERPRAW Check e.
diff --git a/test-suite/ide/undo008.fake b/test-suite/ide/undo008.fake
index 799dc1ac1..1c46c1e87 100644
--- a/test-suite/ide/undo008.fake
+++ b/test-suite/ide/undo008.fake
@@ -15,4 +15,4 @@ INTERP Definition j := O.
INTERP assert True by trivial.
INTERP trivial.
INTERP Qed.
-INTERPRAW Check i. \ No newline at end of file
+INTERPRAW Check i.
diff --git a/test-suite/ide/undo013.fake b/test-suite/ide/undo013.fake
index def2da59e..3b1c61e66 100644
--- a/test-suite/ide/undo013.fake
+++ b/test-suite/ide/undo013.fake
@@ -28,4 +28,4 @@ INTERP apply H.
# </replay>
INTERP Qed.
INTERPRAW Fail idtac.
-INTERPRAW Check (aa,bb,cc). \ No newline at end of file
+INTERPRAW Check (aa,bb,cc).
diff --git a/test-suite/ide/undo014.fake b/test-suite/ide/undo014.fake
index 60897c652..5224b5045 100644
--- a/test-suite/ide/undo014.fake
+++ b/test-suite/ide/undo014.fake
@@ -23,4 +23,4 @@ INTERP Qed.
INTERP apply H.
INTERP Qed.
INTERPRAW Fail idtac.
-INTERPRAW Check (aa,bb,cc). \ No newline at end of file
+INTERPRAW Check (aa,bb,cc).
diff --git a/test-suite/ide/undo015.fake b/test-suite/ide/undo015.fake
index 2bf391051..32e46ec9a 100644
--- a/test-suite/ide/undo015.fake
+++ b/test-suite/ide/undo015.fake
@@ -26,4 +26,4 @@ INTERP Qed.
INTERP apply H.
INTERP Qed.
INTERPRAW Fail idtac.
-INTERPRAW Check (aa,bb,cc). \ No newline at end of file
+INTERPRAW Check (aa,bb,cc).
diff --git a/test-suite/ide/undo016.fake b/test-suite/ide/undo016.fake
index bbc4c578c..2a6e512cb 100644
--- a/test-suite/ide/undo016.fake
+++ b/test-suite/ide/undo016.fake
@@ -31,4 +31,4 @@ INTERP Qed.
INTERP apply H.
INTERP Qed.
INTERPRAW Fail idtac.
-INTERPRAW Check (aa,bb,cc). \ No newline at end of file
+INTERPRAW Check (aa,bb,cc).
diff --git a/test-suite/ide/undo017.fake b/test-suite/ide/undo017.fake
index e5baf6ca6..232360e9d 100644
--- a/test-suite/ide/undo017.fake
+++ b/test-suite/ide/undo017.fake
@@ -10,4 +10,4 @@ REWIND 1
# <replay>
INTERP End M.
# </replay>
-INTERPRAW Check M.x. \ No newline at end of file
+INTERPRAW Check M.x.
diff --git a/test-suite/ide/undo018.fake b/test-suite/ide/undo018.fake
index 42e64218e..ef0945ab5 100644
--- a/test-suite/ide/undo018.fake
+++ b/test-suite/ide/undo018.fake
@@ -10,4 +10,4 @@ REWIND 1
# <replay>
INTERP End M.
# </replay>
-INTERPRAW Check x. \ No newline at end of file
+INTERPRAW Check x.