aboutsummaryrefslogtreecommitdiffstats
path: root/backend/Cmconstr.v
diff options
context:
space:
mode:
Diffstat (limited to 'backend/Cmconstr.v')
-rw-r--r--backend/Cmconstr.v1
1 files changed, 0 insertions, 1 deletions
diff --git a/backend/Cmconstr.v b/backend/Cmconstr.v
index f3a63fae..2cc947c7 100644
--- a/backend/Cmconstr.v
+++ b/backend/Cmconstr.v
@@ -46,7 +46,6 @@ Open Scope cminor_scope.
Fixpoint lift_expr (p: nat) (a: expr) {struct a}: expr :=
match a with
| Evar id => Evar id
- | Eassign id b => Eassign id (lift_expr p b)
| Eop op bl => Eop op (lift_exprlist p bl)
| Eload chunk addr bl => Eload chunk addr (lift_exprlist p bl)
| Estore chunk addr bl c =>