aboutsummaryrefslogtreecommitdiffstats
path: root/riscV/SelectLongproof.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-03-22 10:16:16 +0100
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-03-22 10:16:16 +0100
commit4d53251d4e9a07da1170f4be9b04b5d44381c9ed (patch)
tree6f4ee5c6e54b6c6fcc60311f90bff806d236af97 /riscV/SelectLongproof.v
parent5281141d38a492eea3e080e087b91a314b0be020 (diff)
downloadcompcert-kvx-4d53251d4e9a07da1170f4be9b04b5d44381c9ed.tar.gz
compcert-kvx-4d53251d4e9a07da1170f4be9b04b5d44381c9ed.zip
Risc-V works again (32/64).
Diffstat (limited to 'riscV/SelectLongproof.v')
-rw-r--r--riscV/SelectLongproof.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/riscV/SelectLongproof.v b/riscV/SelectLongproof.v
index 78a1935d..d47b6d64 100644
--- a/riscV/SelectLongproof.v
+++ b/riscV/SelectLongproof.v
@@ -21,6 +21,7 @@ Require Import String Coqlib Maps Integers Floats Errors.
Require Archi.
Require Import AST Values Memory Globalenvs Events.
Require Import Cminor Op CminorSel.
+Require Import OpHelpers OpHelpersproof.
Require Import SelectOp SelectOpproof SplitLong SplitLongproof.
Require Import SelectLong.