summaryrefslogtreecommitdiff
path: root/cfrontend/SimplExprspec.v
diff options
context:
space:
mode:
Diffstat (limited to 'cfrontend/SimplExprspec.v')
-rw-r--r--cfrontend/SimplExprspec.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/cfrontend/SimplExprspec.v b/cfrontend/SimplExprspec.v
index 3f9d7e9..5df0398 100644
--- a/cfrontend/SimplExprspec.v
+++ b/cfrontend/SimplExprspec.v
@@ -20,6 +20,8 @@ Require Import Floats.
Require Import Values.
Require Import Memory.
Require Import AST.
+Require Import Ctypes.
+Require Import Cop.
Require Import Csyntax.
Require Cstrategy.
Require Import Clight.