summaryrefslogtreecommitdiff
path: root/cfrontend/Csem.v
diff options
context:
space:
mode:
authorGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2010-05-10 15:35:02 +0000
committerGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2010-05-10 15:35:02 +0000
commit7999c9ee1f09f7d555e3efc39f030564f76a3354 (patch)
tree6f7937811f9331e3a5f5cdaa59be899c0daf71d3 /cfrontend/Csem.v
parentdf80f5b3745b5d85cbf42601f9532618c063d703 (diff)
- Extended traces so that pointers within globals are supported as event values.
- Revised handling of volatile reads: the execution environment dictates the value read, via the trace of events. git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@1345 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'cfrontend/Csem.v')
-rw-r--r--cfrontend/Csem.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/cfrontend/Csem.v b/cfrontend/Csem.v
index 5f8bbf1..4e4c379 100644
--- a/cfrontend/Csem.v
+++ b/cfrontend/Csem.v
@@ -901,7 +901,7 @@ Inductive step: state -> trace -> state -> Prop :=
E0 (State f f.(fn_body) k e m2)
| step_external_function: forall id targs tres vargs k m vres t m',
- external_call (external_function id targs tres) vargs m t vres m' ->
+ external_call (external_function id targs tres) (Genv.find_symbol ge) vargs m t vres m' ->
step (Callstate (External id targs tres) vargs k m)
t (Returnstate vres k m')
@@ -1106,7 +1106,7 @@ with eval_funcall: mem -> fundef -> list val -> trace -> mem -> val -> Prop :=
Mem.free_list m3 (blocks_of_env e) = Some m4 ->
eval_funcall m (Internal f) vargs t m4 vres
| eval_funcall_external: forall m id targs tres vargs t vres m',
- external_call (external_function id targs tres) vargs m t vres m' ->
+ external_call (external_function id targs tres) (Genv.find_symbol ge) vargs m t vres m' ->
eval_funcall m (External id targs tres) vargs t m' vres.
Scheme exec_stmt_ind2 := Minimality for exec_stmt Sort Prop