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/Tunneling.v | 4 +--- 1 file changed, 1 insertion(+), 3 deletions(-) (limited to 'backend/Tunneling.v') diff --git a/backend/Tunneling.v b/backend/Tunneling.v index fa7ff787..3374d5b4 100644 --- a/backend/Tunneling.v +++ b/backend/Tunneling.v @@ -12,9 +12,7 @@ (** Branch tunneling (optimization of branches to branches). *) -Require Import Coqlib. -Require Import Maps. -Require Import UnionFind. +Require Import Coqlib Maps UnionFind. Require Import AST. Require Import LTL. -- cgit