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/Tailcall.v | 11 ++--------- 1 file changed, 2 insertions(+), 9 deletions(-) (limited to 'backend/Tailcall.v') diff --git a/backend/Tailcall.v b/backend/Tailcall.v index e8ce9e25..939abeea 100644 --- a/backend/Tailcall.v +++ b/backend/Tailcall.v @@ -12,13 +12,7 @@ (** Recognition of tail calls. *) -Require Import Coqlib. -Require Import Maps. -Require Import AST. -Require Import Registers. -Require Import Op. -Require Import RTL. -Require Import Conventions. +Require Import Coqlib Maps AST Registers Op RTL Conventions. (** An [Icall] instruction that stores its result in register [rreg] can be turned into a tail call if: @@ -95,8 +89,7 @@ Definition transf_instr (f: function) (pc: node) (instr: instruction) := end. (** A function is transformed only if its stack block is empty, - as explained above. Moreover, we can turn tail calls off - using a compilation option. *) + as explained above. *) Definition transf_function (f: function) : function := if zeq f.(fn_stacksize) 0 -- cgit