aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
authorGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2015-01-09 11:48:11 +0100
committerGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2015-01-09 11:48:11 +0100
commit0158e2805d29118a818cab11f5c215793bd329ae (patch)
tree9b69de7081aa495ef692a1453871ecfd413cc976 /test-suite
parentf1af234b8b3cc9c6ca0b9d527b660d27a099c866 (diff)
STM: fix handling of side effects in vio2vo
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/Makefile2
-rw-r--r--test-suite/vio/seff.v10
2 files changed, 11 insertions, 1 deletions
diff --git a/test-suite/Makefile b/test-suite/Makefile
index b2f8ad79d..4a3a287c0 100644
--- a/test-suite/Makefile
+++ b/test-suite/Makefile
@@ -435,7 +435,7 @@ vio: $(patsubst %.v,%.vio.log,$(wildcard vio/*.v))
$(HIDE){ \
$(bincoqc) -quick -R vio vio $* 2>&1 && \
$(coqtop) -R vio vio -vio2vo $*.vio 2>&1 && \
- $(bincoqchk) -R vio vio $(subst /,.,$*) 2>&1; \
+ $(bincoqchk) -R vio vio -norec $(subst /,.,$*) 2>&1; \
if [ $$? = 0 ]; then \
echo $(log_success); \
echo " $<...Ok"; \
diff --git a/test-suite/vio/seff.v b/test-suite/vio/seff.v
new file mode 100644
index 000000000..447e77983
--- /dev/null
+++ b/test-suite/vio/seff.v
@@ -0,0 +1,10 @@
+Inductive equal T (x : T) : T -> Type := Equal : equal T x x.
+
+Module bla.
+
+Lemma test n : equal nat n (n + n) -> equal nat (n + n + n) n.
+Proof using.
+intro H. rewrite <- H. rewrite <- H. exact (Equal nat n).
+Qed.
+
+End bla.