From a74f6b45d72834b5b8417297017bd81424123d98 Mon Sep 17 00:00:00 2001 From: xleroy Date: Sun, 7 Mar 2010 15:52:58 +0000 Subject: Merge of the newmem and newextcalls branches: - Revised memory model with concrete representation of ints & floats, and per-byte access permissions - Revised Globalenvs implementation - Matching changes in all languages and proofs. git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@1282 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e --- backend/Tunnelingproof.v | 11 +++++------ 1 file changed, 5 insertions(+), 6 deletions(-) (limited to 'backend/Tunnelingproof.v') diff --git a/backend/Tunnelingproof.v b/backend/Tunnelingproof.v index 92ec68c..4cbcbd4 100644 --- a/backend/Tunnelingproof.v +++ b/backend/Tunnelingproof.v @@ -17,7 +17,7 @@ Require Import Maps. Require Import UnionFind. Require Import AST. Require Import Values. -Require Import Mem. +Require Import Memory. Require Import Events. Require Import Globalenvs. Require Import Smallstep. @@ -348,15 +348,14 @@ Lemma transf_initial_states: exists st2, initial_state tp st2 /\ match_states st1 st2. Proof. intros. inversion H. - exists (Callstate nil (tunnel_fundef f) nil (Genv.init_mem tp)); split. + exists (Callstate nil (tunnel_fundef f) nil m0); split. econstructor; eauto. + apply Genv.init_mem_transf; auto. change (prog_main tp) with (prog_main p). rewrite symbols_preserved. eauto. apply function_ptr_translated; auto. - rewrite <- H2. apply sig_preserved. - replace (Genv.init_mem tp) with (Genv.init_mem p). - constructor. constructor. auto. - symmetry. unfold tp, tunnel_program. apply Genv.init_mem_transf. + rewrite <- H3. apply sig_preserved. + constructor. constructor. Qed. Lemma transf_final_states: -- cgit v1.2.3