summaryrefslogtreecommitdiff
path: root/backend/Tunnelingproof.v
diff options
context:
space:
mode:
authorGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2010-03-07 15:52:58 +0000
committerGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2010-03-07 15:52:58 +0000
commita74f6b45d72834b5b8417297017bd81424123d98 (patch)
treed291cf3f05397658f0fe9d8ecce9b8785a50d270 /backend/Tunnelingproof.v
parent54cba6d4cae1538887f296a62be1c99378fe0916 (diff)
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
Diffstat (limited to 'backend/Tunnelingproof.v')
-rw-r--r--backend/Tunnelingproof.v11
1 files changed, 5 insertions, 6 deletions
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: