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/Constprop.v | 4 ++-- 1 file changed, 2 insertions(+), 2 deletions(-) (limited to 'backend/Constprop.v') diff --git a/backend/Constprop.v b/backend/Constprop.v index 76d8e6ca..d2c4d447 100644 --- a/backend/Constprop.v +++ b/backend/Constprop.v @@ -74,7 +74,7 @@ Definition transf_ros (ae: AE.t) (ros: reg + ident) : reg + ident := Definition const_for_result (a: aval) : option operation := match a with | I n => Some(Ointconst n) - | F n => if generate_float_constants tt then Some(Ofloatconst n) else None + | F n => if Compopts.generate_float_constants tt then Some(Ofloatconst n) else None | Ptr(Gl symb ofs) => Some(Oaddrsymbol symb ofs) | Ptr(Stk ofs) => Some(Oaddrstack ofs) | _ => None @@ -108,7 +108,7 @@ Fixpoint annot_strength_reduction let (targs'', args'') := annot_strength_reduction ae targs' args' in match ty, areg ae arg with | Tint, I n => (AA_int n :: targs'', args'') - | Tfloat, F n => if generate_float_constants tt + | Tfloat, F n => if Compopts.generate_float_constants tt then (AA_float n :: targs'', args'') else (AA_arg ty :: targs'', arg :: args'') | _, _ => (AA_arg ty :: targs'', arg :: args'') -- cgit