From bda5ee25ac991c38f5541a234936f1f6e2226072 Mon Sep 17 00:00:00 2001 From: Xavier Leroy Date: Sun, 16 Nov 2014 18:39:43 +0100 Subject: Add flags to control individual optimization passes + flag -O0 for turning them off. --- backend/Tailcallproof.v | 10 ++++------ 1 file changed, 4 insertions(+), 6 deletions(-) (limited to 'backend/Tailcallproof.v') diff --git a/backend/Tailcallproof.v b/backend/Tailcallproof.v index 1965b18e..cc4ff55e 100644 --- a/backend/Tailcallproof.v +++ b/backend/Tailcallproof.v @@ -13,7 +13,6 @@ (** Recognition of tail calls: correctness proof *) Require Import Coqlib. -Require Import Compopts. Require Import Maps. Require Import AST. Require Import Integers. @@ -183,11 +182,10 @@ Lemma transf_instr_lookup: exists i', (transf_function f).(fn_code)!pc = Some i' /\ transf_instr_spec f i i'. Proof. intros. unfold transf_function. - destruct (zeq (fn_stacksize f) 0). destruct (eliminate_tailcalls tt). + destruct (zeq (fn_stacksize f) 0). simpl. rewrite PTree.gmap. rewrite H. simpl. exists (transf_instr f pc i); split. auto. apply transf_instr_charact; auto. exists i; split. auto. constructor. - exists i; split. auto. constructor. Qed. (** * Semantic properties of the code transformation *) @@ -263,14 +261,14 @@ Lemma sig_preserved: forall f, funsig (transf_fundef f) = funsig f. Proof. destruct f; auto. simpl. unfold transf_function. - destruct (zeq (fn_stacksize f) 0 && eliminate_tailcalls tt); auto. + destruct (zeq (fn_stacksize f) 0); auto. Qed. Lemma stacksize_preserved: forall f, fn_stacksize (transf_function f) = fn_stacksize f. Proof. unfold transf_function. intros. - destruct (zeq (fn_stacksize f) 0 && eliminate_tailcalls tt); auto. + destruct (zeq (fn_stacksize f) 0); auto. Qed. Lemma find_function_translated: @@ -556,7 +554,7 @@ Proof. assert (fn_stacksize (transf_function f) = fn_stacksize f /\ fn_entrypoint (transf_function f) = fn_entrypoint f /\ fn_params (transf_function f) = fn_params f). - unfold transf_function. destruct (zeq (fn_stacksize f) 0 && eliminate_tailcalls tt); auto. + unfold transf_function. destruct (zeq (fn_stacksize f) 0); auto. destruct H0 as [EQ1 [EQ2 EQ3]]. left. econstructor; split. simpl. eapply exec_function_internal; eauto. rewrite EQ1; eauto. -- cgit