From e4723d142aa7b1229cdf5989340342d7c5ce870c Mon Sep 17 00:00:00 2001 From: Xavier Leroy Date: Sun, 6 Mar 2016 10:31:26 +0100 Subject: Update the back-end proofs to the new linking framework. --- backend/Allocation.v | 23 ++++------------------- 1 file changed, 4 insertions(+), 19 deletions(-) (limited to 'backend/Allocation.v') diff --git a/backend/Allocation.v b/backend/Allocation.v index 7534e23f..6a6c1eb6 100644 --- a/backend/Allocation.v +++ b/backend/Allocation.v @@ -12,26 +12,11 @@ (** Register allocation by external oracle and a posteriori validation. *) -Require Import FSets. -Require FSetAVLplus. +Require Import FSets FSetAVLplus. +Require Import Coqlib Ordered Maps Errors Integers Floats. +Require Import AST Lattice Kildall Memdata. Require Archi. -Require Import Coqlib. -Require Import Ordered. -Require Import Errors. -Require Import Maps. -Require Import Lattice. -Require Import AST. -Require Import Integers. -Require Import Floats. -Require Import Memdata. -Require Import Op. -Require Import Registers. -Require Import RTL. -Require Import Kildall. -Require Import Locations. -Require Import Conventions. -Require Import RTLtyping. -Require Import LTL. +Require Import Op Registers RTL Locations Conventions RTLtyping LTL. (** The validation algorithm used here is described in "Validating register allocation and spilling", -- cgit