aboutsummaryrefslogtreecommitdiffstats
path: root/cfrontend/Csem.v
diff options
context:
space:
mode:
authorXavier Leroy <xavier.leroy@inria.fr>2015-02-08 16:41:45 +0100
committerXavier Leroy <xavier.leroy@inria.fr>2015-02-08 16:41:45 +0100
commitf2b1c25aa56a27836652aef3feeee0856c04235c (patch)
tree7eeecd66c8c69f5c17d567a1f8320bec89eff49d /cfrontend/Csem.v
parent30dd68d627f68cca0c2addd006d853379ad720cf (diff)
downloadcompcert-kvx-f2b1c25aa56a27836652aef3feeee0856c04235c.tar.gz
compcert-kvx-f2b1c25aa56a27836652aef3feeee0856c04235c.zip
Interpreter produces more detailed trace, including name of semantic rules used.
Cexec: record names of rules used in every reduction. Interp: print these rule names in -trace mode. Also: simplified the exploration in "-all" mode; give unique names to states. Csem: fix name of reduction rule "red_call".
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 ->