summaryrefslogtreecommitdiff
path: root/backend/InterfGraph.v
diff options
context:
space:
mode:
Diffstat (limited to 'backend/InterfGraph.v')
-rw-r--r--backend/InterfGraph.v6
1 files changed, 1 insertions, 5 deletions
diff --git a/backend/InterfGraph.v b/backend/InterfGraph.v
index 081ef59..8a9dda6 100644
--- a/backend/InterfGraph.v
+++ b/backend/InterfGraph.v
@@ -19,11 +19,6 @@ Require Import Maps.
Require Import Ordered.
Require Import Registers.
Require Import Locations.
-Require Import AST.
-Require Import Op.
-Require Import RTLtyping.
-Require Import RTL.
-Require Import Conventions.
(** Interference graphs are undirected graphs with two kinds of nodes:
- RTL pseudo-registers;
@@ -303,3 +298,4 @@ Proof.
intros. unfold all_interf_regs.
apply in_setregreg_fold'. eapply in_setregmreg_fold. eauto.
Qed.
+