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 --- arm/ConstpropOpproof.v | 14 ++++++++++++++ 1 file changed, 14 insertions(+) (limited to 'arm/ConstpropOpproof.v') diff --git a/arm/ConstpropOpproof.v b/arm/ConstpropOpproof.v index 0e60796a..711bb33b 100644 --- a/arm/ConstpropOpproof.v +++ b/arm/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. @@ -417,6 +418,19 @@ 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. + (* force MATCH to be used *) + assert (val_match_approx (approx_reg app 1%positive) rs#(1%positive)) + by (apply MATCH). + unfold builtin_strength_reduction; intros; simpl; auto. +Qed. + End STRENGTH_REDUCTION. End ANALYSIS. -- cgit