aboutsummaryrefslogtreecommitdiffstats
path: root/cfrontend/Csem.v
diff options
context:
space:
mode:
authorXavier Leroy <xavier.leroy@inria.fr>2015-03-14 10:35:25 +0100
committerXavier Leroy <xavier.leroy@inria.fr>2015-03-14 10:35:25 +0100
commit890141acb930bdb6f985244f81833331382f7b66 (patch)
treecc32d6be06feaebca5076727f5531959e8e37530 /cfrontend/Csem.v
parent67e8b783c7e794d995675a332f118533e6a9b14a (diff)
parent3e01154d693e1c457e1e974f5e9ebaa4601050aa (diff)
downloadcompcert-890141acb930bdb6f985244f81833331382f7b66.tar.gz
compcert-890141acb930bdb6f985244f81833331382f7b66.zip
Merge branch 'master' into struct-passing
Diffstat (limited to 'cfrontend/Csem.v')
-rw-r--r--cfrontend/Csem.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/cfrontend/Csem.v b/cfrontend/Csem.v
index e6e3a321..fafbf29f 100644
--- a/cfrontend/Csem.v
+++ b/cfrontend/Csem.v
@@ -317,7 +317,7 @@ Inductive rred: expr -> mem -> trace -> expr -> mem -> Prop :=
(More exactly, identification of function calls that can reduce.) *)
Inductive callred: expr -> fundef -> list val -> type -> Prop :=
- | red_Ecall: forall vf tyf tyargs tyres cconv el ty fd vargs,
+ | red_call: forall vf tyf tyargs tyres cconv el ty fd vargs,
Genv.find_funct ge vf = Some fd ->
cast_arguments el tyargs vargs ->
type_of_fundef fd = Tfunction tyargs tyres cconv ->