aboutsummaryrefslogtreecommitdiffstats
path: root/backend/Cmconstr.v
diff options
context:
space:
mode:
authorxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2006-09-18 15:52:24 +0000
committerxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2006-09-18 15:52:24 +0000
commit165407527b1be7df6a376791719321c788e55149 (patch)
tree35c2eb9603f007b033fced56f21fa49fd105562f /backend/Cmconstr.v
parent1346309fd03e19da52156a700d037c348f27af0d (diff)
downloadcompcert-165407527b1be7df6a376791719321c788e55149.tar.gz
compcert-165407527b1be7df6a376791719321c788e55149.zip
Simplification de Cminor: les affectations de variables locales ne sont
plus des expressions mais des statements (Eassign -> Sassign). Cela simplifie les preuves et ameliore la qualite du RTL produit. git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@111 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
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 =>