summaryrefslogtreecommitdiff
path: root/cfrontend/Cexec.v
diff options
context:
space:
mode:
Diffstat (limited to 'cfrontend/Cexec.v')
-rw-r--r--cfrontend/Cexec.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/cfrontend/Cexec.v b/cfrontend/Cexec.v
index bc85efd..b41902c 100644
--- a/cfrontend/Cexec.v
+++ b/cfrontend/Cexec.v
@@ -863,7 +863,7 @@ Fixpoint step_expr (k: kind) (a: expr) (m: mem): reducts expr :=
let op := match id with Incr => Oadd | Decr => Osub end in
let r' :=
Ecomma (Eassign (Eloc b ofs ty)
- (Ebinop op (Eval v1 ty) (Eval (Vint Int.one) type_int32s) (typeconv ty))
+ (Ebinop op (Eval v1 ty) (Eval (Vint Int.one) type_int32s) (incrdecr_type ty))
ty)
(Eval v1 ty) ty in
topred (Rred r' m t)