aboutsummaryrefslogtreecommitdiffstats
path: root/cfrontend/Clight.v
diff options
context:
space:
mode:
authorXavier Leroy <xavierleroy@users.noreply.github.com>2015-04-01 18:27:15 +0200
committerXavier Leroy <xavierleroy@users.noreply.github.com>2015-04-01 18:27:15 +0200
commit68e2ce02f8d69b26c9cea6e0d338f855cbea3ace (patch)
tree98acb09c398112bff31ce34c0857aa0f4e9b8e23 /cfrontend/Clight.v
parent5d6febecb8c0f90a627033744f6f62164645a1a4 (diff)
parentdaccc2928e6410c4e8c886ea7d019fd9a071b931 (diff)
downloadcompcert-68e2ce02f8d69b26c9cea6e0d338f855cbea3ace.tar.gz
compcert-68e2ce02f8d69b26c9cea6e0d338f855cbea3ace.zip
Merge pull request #31 from AbsInt/null-ptr-cmp
Revised semantics of comparisons between a pointer and 0.
Diffstat (limited to 'cfrontend/Clight.v')
-rw-r--r--cfrontend/Clight.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/cfrontend/Clight.v b/cfrontend/Clight.v
index 7a45b453..77511b2c 100644
--- a/cfrontend/Clight.v
+++ b/cfrontend/Clight.v
@@ -403,7 +403,7 @@ Inductive eval_expr: expr -> val -> Prop :=
eval_expr (Eaddrof a ty) (Vptr loc ofs)
| eval_Eunop: forall op a ty v1 v,
eval_expr a v1 ->
- sem_unary_operation op v1 (typeof a) = Some v ->
+ sem_unary_operation op v1 (typeof a) m = Some v ->
eval_expr (Eunop op a ty) v
| eval_Ebinop: forall op a1 a2 ty v1 v2 v,
eval_expr a1 v1 ->
@@ -620,7 +620,7 @@ Inductive step: state -> trace -> state -> Prop :=
| step_ifthenelse: forall f a s1 s2 k e le m v1 b,
eval_expr e le m a v1 ->
- bool_val v1 (typeof a) = Some b ->
+ bool_val v1 (typeof a) m = Some b ->
step (State f (Sifthenelse a s1 s2) k e le m)
E0 (State f (if b then s1 else s2) k e le m)