aboutsummaryrefslogtreecommitdiffstats
path: root/backend/Allocproof.v
diff options
context:
space:
mode:
Diffstat (limited to 'backend/Allocproof.v')
-rw-r--r--backend/Allocproof.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/backend/Allocproof.v b/backend/Allocproof.v
index 6c10d27f..29dbcbe8 100644
--- a/backend/Allocproof.v
+++ b/backend/Allocproof.v
@@ -13,6 +13,7 @@
(** Correctness proof for the [Allocation] pass (validated translation from
RTL to LTL). *)
+Require Import FunInd.
Require Import FSets.
Require Import Coqlib Ordered Maps Errors Integers Floats.
Require Import AST Linking Lattice Kildall.