aboutsummaryrefslogtreecommitdiffstats
path: root/arm/SelectLong.vp
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-03-22 09:51:56 +0100
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-03-22 09:51:56 +0100
commit5281141d38a492eea3e080e087b91a314b0be020 (patch)
treec27e1da95d37abc1a14839c0bfb26fd2dd102077 /arm/SelectLong.vp
parent1fd8a013a4fa57fcfa6c9e295638871153e596ee (diff)
downloadcompcert-kvx-5281141d38a492eea3e080e087b91a314b0be020.tar.gz
compcert-kvx-5281141d38a492eea3e080e087b91a314b0be020.zip
ARM repasse
Diffstat (limited to 'arm/SelectLong.vp')
-rw-r--r--arm/SelectLong.vp2
1 files changed, 1 insertions, 1 deletions
diff --git a/arm/SelectLong.vp b/arm/SelectLong.vp
index cc7a38f6..b4cdd0e3 100644
--- a/arm/SelectLong.vp
+++ b/arm/SelectLong.vp
@@ -16,6 +16,6 @@ Require Import Coqlib.
Require Import Compopts.
Require Import AST Integers Floats.
Require Import Op CminorSel.
-Require Import SelectOp SplitLong.
+Require Import OpHelpers SelectOp SplitLong.
(** This file is empty because we use the default implementation provided in [SplitLong]. *)