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/Constpropproof.v | 5 +++-- 1 file changed, 3 insertions(+), 2 deletions(-) (limited to 'backend/Constpropproof.v') diff --git a/backend/Constpropproof.v b/backend/Constpropproof.v index 41afe8c8..d88d6e43 100644 --- a/backend/Constpropproof.v +++ b/backend/Constpropproof.v @@ -14,6 +14,7 @@ Require Import Coqlib. Require Import Maps. +Require Compopts. Require Import AST. Require Import Integers. Require Import Values. @@ -157,7 +158,7 @@ Proof. - (* integer *) inv H. inv H0. exists (Vint n); auto. - (* float *) - destruct (generate_float_constants tt); inv H. inv H0. exists (Vfloat f); auto. + destruct (Compopts.generate_float_constants tt); inv H. inv H0. exists (Vfloat f); auto. - (* pointer *) destruct p; try discriminate. + (* global *) @@ -235,7 +236,7 @@ Proof. * exists eargs''; split; auto; simpl; f_equal; auto. generalize (MATCH arg); fold (areg ae arg); rewrite E2; intros VM. inv VM. rewrite <- H0 in *. inv H5; auto. - * destruct (generate_float_constants tt); inv H1; auto. + * destruct (Compopts.generate_float_constants tt); inv H1; auto. exists eargs''; split; auto; simpl; f_equal; auto. generalize (MATCH arg); fold (areg ae arg); rewrite E2; intros VM. inv VM. rewrite <- H0 in *. inv H5; auto. -- cgit