aboutsummaryrefslogtreecommitdiffstats
path: root/x86/CombineOpproof.v
diff options
context:
space:
mode:
Diffstat (limited to 'x86/CombineOpproof.v')
-rw-r--r--x86/CombineOpproof.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/x86/CombineOpproof.v b/x86/CombineOpproof.v
index a7024501..69abbf61 100644
--- a/x86/CombineOpproof.v
+++ b/x86/CombineOpproof.v
@@ -13,6 +13,7 @@
(** Recognition of combined operations, addressing modes and conditions
during the [CSE] phase. *)
+Require Import FunInd.
Require Import Coqlib.
Require Import Integers Values Memory.
Require Import Op RTL CSEdomain.