aboutsummaryrefslogtreecommitdiffstats
path: root/arm/Selection.v
diff options
context:
space:
mode:
Diffstat (limited to 'arm/Selection.v')
-rw-r--r--arm/Selection.v1
1 files changed, 0 insertions, 1 deletions
diff --git a/arm/Selection.v b/arm/Selection.v
index 1b5411b1..d04a4ca3 100644
--- a/arm/Selection.v
+++ b/arm/Selection.v
@@ -1359,7 +1359,6 @@ Fixpoint sel_stmt (s: Cminor.stmt) : stmt :=
Scall optid sg (sel_expr fn) (sel_exprlist args)
| Cminor.Stailcall sg fn args =>
Stailcall sg (sel_expr fn) (sel_exprlist args)
- | Cminor.Salloc id b => Salloc id (sel_expr b)
| Cminor.Sseq s1 s2 => Sseq (sel_stmt s1) (sel_stmt s2)
| Cminor.Sifthenelse e ifso ifnot =>
Sifthenelse (condexpr_of_expr (sel_expr e))