summaryrefslogtreecommitdiff
path: root/cfrontend/Csharpminor.v
diff options
context:
space:
mode:
authorGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2010-05-23 15:26:33 +0000
committerGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2010-05-23 15:26:33 +0000
commit3a050b22f37f3c79a10a8ebae3d292fa77e91b76 (patch)
tree16a0d9366f6805cfc9726c0b80dd8da84cb63a3d /cfrontend/Csharpminor.v
parent7999c9ee1f09f7d555e3efc39f030564f76a3354 (diff)
More faithful semantics for volatile reads and writes.
git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@1346 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'cfrontend/Csharpminor.v')
-rw-r--r--cfrontend/Csharpminor.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/cfrontend/Csharpminor.v b/cfrontend/Csharpminor.v
index 4c61918..558ae1c 100644
--- a/cfrontend/Csharpminor.v
+++ b/cfrontend/Csharpminor.v
@@ -516,7 +516,7 @@ Inductive step: state -> trace -> state -> Prop :=
E0 (State f f.(fn_body) k e m2)
| step_external_function: forall ef vargs k m t vres m',
- external_call ef (Genv.find_symbol ge) vargs m t vres m' ->
+ external_call ef ge vargs m t vres m' ->
step (Callstate (External ef) vargs k m)
t (Returnstate vres k m')
@@ -554,7 +554,7 @@ Inductive final_state: state -> int -> Prop :=
Definition global_var_env (p: program): gvarenv :=
List.fold_left
- (fun gve x => match x with (id, init, k) => PTree.set id k gve end)
+ (fun gve x => match x with (id, v) => PTree.set id (gvar_info v) gve end)
p.(prog_vars) (PTree.empty var_kind).
Definition exec_program (p: program) (beh: program_behavior) : Prop :=