summaryrefslogtreecommitdiff
path: root/cfrontend/SimplExpr.v
diff options
context:
space:
mode:
Diffstat (limited to 'cfrontend/SimplExpr.v')
-rw-r--r--cfrontend/SimplExpr.v9
1 files changed, 4 insertions, 5 deletions
diff --git a/cfrontend/SimplExpr.v b/cfrontend/SimplExpr.v
index 854d345..1ead0ae 100644
--- a/cfrontend/SimplExpr.v
+++ b/cfrontend/SimplExpr.v
@@ -488,13 +488,12 @@ Fixpoint transl_stmt (s: Csyntax.statement) : mon statement :=
with transl_lblstmt (ls: Csyntax.labeled_statements) : mon labeled_statements :=
match ls with
- | Csyntax.LSdefault s =>
- do ts <- transl_stmt s;
- ret (LSdefault ts)
- | Csyntax.LScase n s ls1 =>
+ | Csyntax.LSnil =>
+ ret LSnil
+ | Csyntax.LScons c s ls1 =>
do ts <- transl_stmt s;
do tls1 <- transl_lblstmt ls1;
- ret (LScase n ts tls1)
+ ret (LScons c ts tls1)
end.
(** Translation of a function *)