aboutsummaryrefslogtreecommitdiffstats
path: root/mppa_k1c/SelectLongproof.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-03-22 09:27:40 +0100
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2019-03-22 09:27:40 +0100
commit1fd8a013a4fa57fcfa6c9e295638871153e596ee (patch)
tree1068e03e029a186543ff653b4a539bf91948c60e /mppa_k1c/SelectLongproof.v
parent5a425ba34f3f2520de752ea95a4636a9437c312a (diff)
downloadcompcert-kvx-1fd8a013a4fa57fcfa6c9e295638871153e596ee.tar.gz
compcert-kvx-1fd8a013a4fa57fcfa6c9e295638871153e596ee.zip
restructuration pour compilation toute archi
Diffstat (limited to 'mppa_k1c/SelectLongproof.v')
-rw-r--r--mppa_k1c/SelectLongproof.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/mppa_k1c/SelectLongproof.v b/mppa_k1c/SelectLongproof.v
index 4723278a..79187338 100644
--- a/mppa_k1c/SelectLongproof.v
+++ b/mppa_k1c/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.