summaryrefslogtreecommitdiff
path: root/cfrontend/Csem.v
diff options
context:
space:
mode:
authorGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2007-10-17 08:55:50 +0000
committerGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2007-10-17 08:55:50 +0000
commit0d2f4a416abcc44fb000758a134a38562a5d6d19 (patch)
treebd2b6bcb822a7b30fec5a59cf5b448389dfcf307 /cfrontend/Csem.v
parent8a07279be78b9e504d0ea304bca72c49fdad0b37 (diff)
Relaxation de la regle d'evaluation Ecast
git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@420 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 af601ac..8d8f88a 100644
--- a/cfrontend/Csem.v
+++ b/cfrontend/Csem.v
@@ -562,10 +562,10 @@ Inductive eval_expr: expr -> val -> Prop :=
eval_expr a2 v2 ->
bool_of_val v2 (typeof a2) v ->
eval_expr (Expr (Eandbool a1 a2) ty) v
- | eval_Ecast: forall a ty v1 v,
+ | eval_Ecast: forall a ty ty' v1 v,
eval_expr a v1 ->
cast v1 (typeof a) ty v ->
- eval_expr (Expr (Ecast ty a) ty) v
+ eval_expr (Expr (Ecast ty a) ty') v
(** [eval_lvalue ge e m a b ofs] defines the evaluation of expression [a]
in l-value position. The result is the memory location [b, ofs]