aboutsummaryrefslogtreecommitdiffstats
path: root/cfrontend/Csharpminor.v
diff options
context:
space:
mode:
Diffstat (limited to 'cfrontend/Csharpminor.v')
-rw-r--r--cfrontend/Csharpminor.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/cfrontend/Csharpminor.v b/cfrontend/Csharpminor.v
index e42091af..4393640c 100644
--- a/cfrontend/Csharpminor.v
+++ b/cfrontend/Csharpminor.v
@@ -321,7 +321,7 @@ Inductive eval_expr: expr -> val -> Prop :=
eval_expr (Evar id) v
| eval_Eaddrof: forall id b,
eval_var_addr e id b ->
- eval_expr (Eaddrof id) (Vptr b Int.zero)
+ eval_expr (Eaddrof id) (Vptr b Ptrofs.zero)
| eval_Econst: forall cst v,
eval_constant cst = Some v ->
eval_expr (Econst cst) v