From c4877832826fa26aea9c236f16bdc2de16c98150 Mon Sep 17 00:00:00 2001 From: xleroy Date: Sun, 15 Jan 2012 08:57:09 +0000 Subject: Added volatile_read_global and volatile_store_global builtins. Finished updating IA32 and ARM ports. git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@1792 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e --- powerpc/ConstpropOpproof.v | 19 +++++++++++++++++++ 1 file changed, 19 insertions(+) (limited to 'powerpc/ConstpropOpproof.v') diff --git a/powerpc/ConstpropOpproof.v b/powerpc/ConstpropOpproof.v index 36444b3e..3b5021e2 100644 --- a/powerpc/ConstpropOpproof.v +++ b/powerpc/ConstpropOpproof.v @@ -19,6 +19,7 @@ Require Import Floats. Require Import Values. Require Import Memory. Require Import Globalenvs. +Require Import Events. Require Import Op. Require Import Registers. Require Import RTL. @@ -404,6 +405,24 @@ Proof. auto. Qed. +Lemma builtin_strength_reduction_correct: + forall ef args vl m t vres m', + vl = approx_regs app args -> + external_call ef ge rs##args m t vres m' -> + let (ef', args') := builtin_strength_reduction ef args vl in + external_call ef' ge rs##args' m t vres m'. +Proof. + intros until m'. unfold builtin_strength_reduction. + destruct (builtin_strength_reduction_match ef args vl); simpl; intros; InvApproxRegs; SimplVMA. + unfold symbol_address in H. destruct (Genv.find_symbol ge symb) as [b|]_eqn; rewrite H in H0. + rewrite volatile_load_global_charact. exists b; auto. + inv H0. + unfold symbol_address in H1. destruct (Genv.find_symbol ge symb) as [b|]_eqn; rewrite H1 in H0. + rewrite volatile_store_global_charact. exists b; auto. + inv H0. + auto. +Qed. + End STRENGTH_REDUCTION. End ANALYSIS. -- cgit