aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/vio
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/vio
parentf1af234b8b3cc9c6ca0b9d527b660d27a099c866 (diff)
STM: fix handling of side effects in vio2vo
Diffstat (limited to 'test-suite/vio')
-rw-r--r--test-suite/vio/seff.v10
1 files changed, 10 insertions, 0 deletions
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.