aboutsummaryrefslogtreecommitdiffstats
path: root/arm/SelectOp.vp
diff options
context:
space:
mode:
authorxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2014-05-28 14:55:10 +0000
committerxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2014-05-28 14:55:10 +0000
commitc8a892a09e9f61c3af7dae30d39509558f77462a (patch)
tree639ce60c2a12ed974e005a9a4f267b8116455354 /arm/SelectOp.vp
parent3fa79790e617d87584598746296e626e0ce3b256 (diff)
downloadcompcert-kvx-c8a892a09e9f61c3af7dae30d39509558f77462a.tar.gz
compcert-kvx-c8a892a09e9f61c3af7dae30d39509558f77462a.zip
Instead of having two expansions of shrximm (one in SelectOp, one in Asmgen), move the most efficient expansion to Asmgen.
git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@2504 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'arm/SelectOp.vp')
-rw-r--r--arm/SelectOp.vp9
1 files changed, 1 insertions, 8 deletions
diff --git a/arm/SelectOp.vp b/arm/SelectOp.vp
index efd9e482..e4005c92 100644
--- a/arm/SelectOp.vp
+++ b/arm/SelectOp.vp
@@ -291,14 +291,7 @@ Definition divu_base (e1: expr) (e2: expr) := Eop Odivu (e1:::e2:::Enil).
Definition modu_base := mod_aux Odivu.
Definition shrximm (e1: expr) (n2: int) :=
- if Int.eq n2 Int.zero
- then e1
- else Elet e1
- (shrimm
- (add (Eletvar O)
- (shruimm (shrimm (Eletvar O) (Int.repr 31))
- (Int.sub Int.iwordsize n2)))
- n2).
+ if Int.eq n2 Int.zero then e1 else Eop (Oshrximm n2) (e1:::Enil).
(** ** General shifts *)