From 3ec022950ec233a2af418aacd1755fce4d701724 Mon Sep 17 00:00:00 2001 From: xleroy Date: Wed, 19 Feb 2014 09:55:45 +0000 Subject: Add option -Os to optimize for code size rather than for execution speed. Refactored compilation flags that affect the Coq part (module Compopts). Added support for C99 for loops with declarations. git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@2410 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e --- backend/Tailcall.v | 3 +-- 1 file changed, 1 insertion(+), 2 deletions(-) (limited to 'backend/Tailcall.v') diff --git a/backend/Tailcall.v b/backend/Tailcall.v index 26beb340..25da531c 100644 --- a/backend/Tailcall.v +++ b/backend/Tailcall.v @@ -14,6 +14,7 @@ Require Import Coqlib. Require Import Maps. +Require Import Compopts. Require Import AST. Require Import Registers. Require Import Op. @@ -98,8 +99,6 @@ Definition transf_instr (f: function) (pc: node) (instr: instruction) := as explained above. Moreover, we can turn tail calls off using a compilation option. *) -Parameter eliminate_tailcalls: unit -> bool. - Definition transf_function (f: function) : function := if zeq f.(fn_stacksize) 0 && eliminate_tailcalls tt then RTL.transf_function (transf_instr f) f -- cgit