[project @ 1996-04-08 16:15:43 by partain]
[ghc-hetmet.git] / ghc / compiler / simplCore / Simplify.lhs
1 %
2 % (c) The AQUA Project, Glasgow University, 1993-1996
3 %
4 \section[Simplify]{The main module of the simplifier}
5
6 \begin{code}
7 #include "HsVersions.h"
8
9 module Simplify ( simplTopBinds, simplExpr, simplBind ) where
10
11 import Ubiq{-uitous-}
12 import SmplLoop         -- paranoia checking
13
14 import BinderInfo
15 import CmdLineOpts      ( SimplifierSwitch(..) )
16 import ConFold          ( completePrim )
17 import CoreSyn
18 import CoreUtils        ( coreExprType, nonErrorRHSs, maybeErrorApp,
19                           unTagBinders, squashableDictishCcExpr,
20                           manifestlyWHNF
21                         )
22 import Id               ( idType, idWantsToBeINLINEd,
23                           getIdDemandInfo, addIdDemandInfo,
24                           GenId{-instance NamedThing-}
25                         )
26 import IdInfo           ( willBeDemanded, DemandInfo )
27 import Literal          ( isNoRepLit )
28 import Maybes           ( maybeToBool )
29 import Name             ( isLocallyDefined )
30 import PprStyle         ( PprStyle(..) )
31 import PprType          ( GenType{-instance Outputable-} )
32 import PrelInfo         ( realWorldStateTy )
33 import Pretty           ( ppAbove )
34 import PrimOp           ( primOpOkForSpeculation, PrimOp(..) )
35 import SimplCase        ( simplCase, bindLargeRhs )
36 import SimplEnv
37 import SimplMonad
38 import SimplVar         ( completeVar )
39 import SimplUtils
40 import Type             ( mkTyVarTy, mkTyVarTys, mkAppTy,
41                           splitFunTy, getFunTy_maybe, eqTy
42                         )
43 import Util             ( isSingleton, panic, pprPanic, assertPanic )
44 \end{code}
45
46 The controlling flags, and what they do
47 ~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
48
49 passes:
50 ------
51 -fsimplify              = run the simplifier
52 -ffloat-inwards         = runs the float lets inwards pass
53 -ffloat                 = runs the full laziness pass
54                           (ToDo: rename to -ffull-laziness)
55 -fupdate-analysis       = runs update analyser
56 -fstrictness            = runs strictness analyser
57 -fsaturate-apps         = saturates applications (eta expansion)
58
59 options:
60 -------
61 -ffloat-past-lambda     = OK to do full laziness.
62                           (ToDo: remove, as the full laziness pass is
63                                  useless without this flag, therefore
64                                  it is unnecessary. Just -ffull-laziness
65                                  should be kept.)
66
67 -ffloat-lets-ok         = OK to float lets out of lets if the enclosing
68                           let is strict or if the floating will expose
69                           a WHNF [simplifier].
70
71 -ffloat-primops-ok      = OK to float out of lets cases whose scrutinee
72                           is a primop that cannot fail [simplifier].
73
74 -fcode-duplication-ok   = allows the previous option to work on cases with
75                           multiple branches [simplifier].
76
77 -flet-to-case           = does let-to-case transformation [simplifier].
78
79 -fcase-of-case          = does case of case transformation [simplifier].
80
81 -fpedantic-bottoms      = does not allow:
82                              case x of y -> e  ===>  e[x/y]
83                           (which may turn bottom into non-bottom)
84
85
86                         NOTES ON INLINING
87                         ~~~~~~~~~~~~~~~~~
88
89 Inlining is one of the delicate aspects of the simplifier.  By
90 ``inlining'' we mean replacing an occurrence of a variable ``x'' by
91 the RHS of x's definition.  Thus
92
93         let x = e in ...x...    ===>   let x = e in ...e...
94
95 We have two mechanisms for inlining:
96
97 1.  Unconditional.  The occurrence analyser has pinned an (OneOcc
98 FunOcc NoDupDanger NotInsideSCC n) flag on the variable, saying ``it's
99 certainly safe to inline this variable, and to drop its binding''.
100 (...Umm... if n <= 1; if n > 1, it is still safe, provided you are
101 happy to be duplicating code...) When it encounters such a beast, the
102 simplifer binds the variable to its RHS (in the id_env) and continues.
103 It doesn't even look at the RHS at that stage.  It also drops the
104 binding altogether.
105
106 2.  Conditional.  In all other situations, the simplifer simplifies
107 the RHS anyway, and keeps the new binding.  It also binds the new
108 (cloned) variable to a ``suitable'' UnfoldingDetails in the UnfoldEnv.
109
110 Here, ``suitable'' might mean NoUnfoldingDetails (if the occurrence
111 info is ManyOcc and the RHS is not a manifest HNF, or UnfoldAlways (if
112 the variable has an INLINE pragma on it).  The idea is that anything
113 in the UnfoldEnv is safe to use, but also has an enclosing binding if
114 you decide not to use it.
115
116 Head normal forms
117 ~~~~~~~~~~~~~~~~~
118 We *never* put a non-HNF unfolding in the UnfoldEnv except in the
119 INLINE-pragma case.
120
121 At one time I thought it would be OK to put non-HNF unfoldings in for
122 variables which occur only once [if they got inlined at that
123 occurrence the RHS of the binding would become dead, so no duplication
124 would occur].   But consider:
125 @
126         let x = <expensive>
127             f = \y -> ...y...y...y...
128         in f x
129 @
130 Now, it seems that @x@ appears only once, but even so it is NOT safe
131 to put @x@ in the UnfoldEnv, because @f@ will be inlined, and will
132 duplicate the references to @x@.
133
134 Because of this, the "unconditional-inline" mechanism above is the
135 only way in which non-HNFs can get inlined.
136
137 INLINE pragmas
138 ~~~~~~~~~~~~~~
139
140 When a variable has an INLINE pragma on it --- which includes wrappers
141 produced by the strictness analyser --- we treat it rather carefully.
142
143 For a start, we are careful not to substitute into its RHS, because
144 that might make it BIG, and the user said "inline exactly this", not
145 "inline whatever you get after inlining other stuff inside me".  For
146 example
147
148         let f = BIG
149         in {-# INLINE y #-} y = f 3
150         in ...y...y...
151
152 Here we don't want to substitute BIG for the (single) occurrence of f,
153 because then we'd duplicate BIG when we inline'd y.  (Exception:
154 things in the UnfoldEnv with UnfoldAlways flags, which originated in
155 other INLINE pragmas.)
156
157 So, we clean out the UnfoldEnv of all GenForm inlinings before
158 going into such an RHS.
159
160 What about imports?  They don't really matter much because we only
161 inline relatively small things via imports.
162
163 We augment the the UnfoldEnv with UnfoldAlways guidance if there's an
164 INLINE pragma.  We also do this for the RHSs of recursive decls,
165 before looking at the recursive decls. That way we achieve the effect
166 of inlining a wrapper in the body of its worker, in the case of a
167 mutually-recursive worker/wrapper split.
168
169
170 %************************************************************************
171 %*                                                                      *
172 \subsection[Simplify-simplExpr]{The main function: simplExpr}
173 %*                                                                      *
174 %************************************************************************
175
176 At the top level things are a little different.
177
178   * No cloning (not allowed for exported Ids, unnecessary for the others)
179
180   * No floating.   Case floating is obviously out.  Let floating is
181         theoretically OK, but dangerous because of space leaks.
182         The long-distance let-floater lifts these lets.
183
184 \begin{code}
185 simplTopBinds :: SimplEnv -> [InBinding] -> SmplM [OutBinding]
186
187 simplTopBinds env [] = returnSmpl []
188
189 -- Dead code is now discarded by the occurrence analyser,
190
191 simplTopBinds env (NonRec binder@(in_id, occ_info) rhs : binds)
192   | inlineUnconditionally ok_to_dup_code occ_info
193   = let
194         new_env = extendIdEnvWithInlining env env binder rhs
195     in
196     simplTopBinds new_env binds
197   where
198     ok_to_dup_code = switchIsSet env SimplOkToDupCode
199
200 simplTopBinds env (NonRec binder@(in_id,occ_info) rhs : binds)
201   =     -- No cloning necessary at top level
202         -- Process the binding
203     simplRhsExpr env binder rhs         `thenSmpl` \ rhs' ->
204     let
205        new_env = case rhs' of
206          Var v                      -> extendIdEnvWithAtom env binder (VarArg v)
207          Lit i | not (isNoRepLit i) -> extendIdEnvWithAtom env binder (LitArg i)
208          other                      -> extendUnfoldEnvGivenRhs env binder in_id rhs'
209     in
210         -- Process the other bindings
211     simplTopBinds new_env binds `thenSmpl` \ binds' ->
212
213         -- Glue together and return ...
214         -- We leave it to susequent occurrence analysis to throw away
215         -- an unused atom binding. This localises the decision about
216         -- discarding top-level bindings.
217     returnSmpl (NonRec in_id rhs' : binds')
218
219 simplTopBinds env (Rec pairs : binds)
220   = simplRecursiveGroup env triples     `thenSmpl` \ (bind', new_env) ->
221
222         -- Process the other bindings
223     simplTopBinds new_env binds         `thenSmpl` \ binds' ->
224
225         -- Glue together and return
226     returnSmpl (bind' : binds')
227   where
228     triples = [(id, (binder, rhs)) | (binder@(id,_), rhs) <- pairs]
229                 -- No cloning necessary at top level
230 \end{code}
231
232 %************************************************************************
233 %*                                                                      *
234 \subsection[Simplify-simplExpr]{The main function: simplExpr}
235 %*                                                                      *
236 %************************************************************************
237
238
239 \begin{code}
240 simplExpr :: SimplEnv
241           -> InExpr -> [OutArg]
242           -> SmplM OutExpr
243 \end{code}
244
245 The expression returned has the same meaning as the input expression
246 applied to the specified arguments.
247
248
249 Variables
250 ~~~~~~~~~
251 Check if there's a macro-expansion, and if so rattle on.  Otherwise do
252 the more sophisticated stuff.
253
254 \begin{code}
255 simplExpr env (Var v) args
256   = case (lookupId env v) of
257       Nothing -> let
258                     new_v = simplTyInId env v
259                  in
260                  completeVar env new_v args
261
262       Just info ->
263         case info of
264           ItsAnAtom (LitArg lit)        -- A boring old literal
265                         -- Paranoia check for args empty
266             ->  case args of
267                   []    -> returnSmpl (Lit lit)
268                   other -> panic "simplExpr:coVar"
269
270           ItsAnAtom (VarArg var)        -- More interesting!  An id!
271                                         -- No need to substitute the type env here,
272                                         -- because we already have!
273             -> completeVar env var args
274
275           InlineIt id_env ty_env in_expr        -- A macro-expansion
276             -> simplExpr (replaceInEnvs env (ty_env, id_env)) in_expr args
277 \end{code}
278
279 Literals
280 ~~~~~~~~
281
282 \begin{code}
283 simplExpr env (Lit l) [] = returnSmpl (Lit l)
284 #ifdef DEBUG
285 simplExpr env (Lit l) _  = panic "simplExpr:Lit with argument"
286 #endif
287 \end{code}
288
289 Primitive applications are simple.
290 ~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
291
292 NB: Prim expects an empty argument list! (Because it should be
293 saturated and not higher-order. ADR)
294
295 \begin{code}
296 simplExpr env (Prim op prim_args) args
297   = ASSERT (null args)
298     let
299         prim_args' = [simplArg env prim_arg | prim_arg <- prim_args]
300         op'        = simpl_op op
301     in
302     completePrim env op' prim_args'
303   where
304     -- PrimOps just need any types in them renamed.
305
306     simpl_op (CCallOp label is_asm may_gc arg_tys result_ty)
307       = let
308             arg_tys'    = map (simplTy env) arg_tys
309             result_ty'  = simplTy env result_ty
310         in
311         CCallOp label is_asm may_gc arg_tys' result_ty'
312
313     simpl_op other_op = other_op
314 \end{code}
315
316 Constructor applications
317 ~~~~~~~~~~~~~~~~~~~~~~~~
318 Nothing to try here.  We only reuse constructors when they appear as the
319 rhs of a let binding (see completeLetBinding).
320
321 \begin{code}
322 simplExpr env (Con con con_args) args
323   = ASSERT( null args )
324     returnSmpl (Con con [simplArg env con_arg | con_arg <- con_args])
325 \end{code}
326
327
328 Applications are easy too:
329 ~~~~~~~~~~~~~~~~~~~~~~~~~~
330 Just stuff 'em in the arg stack
331
332 \begin{code}
333 simplExpr env (App fun arg) args
334   = simplExpr env fun (simplArg env arg : args)
335 \end{code}
336
337 Type lambdas
338 ~~~~~~~~~~~~
339
340 We only eta-reduce a type lambda if all type arguments in the body can
341 be eta-reduced. This requires us to collect up all tyvar parameters so
342 we can pass them all to @mkTyLamTryingEta@.
343
344 \begin{code}
345 simplExpr env (Lam (TyBinder tyvar) body) (TyArg ty : args)
346   = -- ASSERT(not (isPrimType ty))
347     let
348         new_env = extendTyEnv env tyvar ty
349     in
350     tick TyBetaReduction        `thenSmpl_`
351     simplExpr new_env body args
352
353 simplExpr env tylam@(Lam (TyBinder tyvar) body) []
354   = do_tylambdas env [] tylam
355   where
356     do_tylambdas env tyvars' (Lam (TyBinder tyvar) body)
357       =   -- Clone the type variable
358         cloneTyVarSmpl tyvar            `thenSmpl` \ tyvar' ->
359         let
360             new_env = extendTyEnv env tyvar (mkTyVarTy tyvar')
361         in
362         do_tylambdas new_env (tyvar':tyvars') body
363
364     do_tylambdas env tyvars' body
365       = simplExpr env body []           `thenSmpl` \ body' ->
366         returnSmpl (
367            (if switchIsSet env SimplDoEtaReduction
368            then mkTyLamTryingEta
369            else mkTyLam) (reverse tyvars')  body'
370         )
371
372 #ifdef DEBUG
373 simplExpr env (Lam (TyBinder _) _) (_ : _)
374   = panic "simplExpr:TyLam with non-TyArg"
375 #endif
376 \end{code}
377
378
379 Ordinary lambdas
380 ~~~~~~~~~~~~~~~~
381
382 \begin{code}
383 simplExpr env (Lam (ValBinder binder) body) args
384   | null leftover_binders
385   =     -- The lambda is saturated (or over-saturated)
386     tick BetaReduction  `thenSmpl_`
387     simplExpr env_for_enough_args body leftover_args
388
389   | otherwise
390   =     -- Too few args to saturate the lambda
391     ASSERT( null leftover_args )
392
393     (if not (null args) -- ah, we must've gotten rid of some...
394      then tick BetaReduction
395      else returnSmpl (panic "BetaReduction")
396     ) `thenSmpl_`
397
398     simplLam env_for_too_few_args leftover_binders body
399              0 {- Guaranteed applied to at least 0 args! -}
400
401   where
402     (binder_args_pairs, leftover_binders, leftover_args) = collect_val_args binder args
403
404     env_for_enough_args  = extendIdEnvWithAtomList env binder_args_pairs
405
406     env_for_too_few_args = extendIdEnvWithAtomList env zapped_binder_args_pairs
407
408         -- Since there aren't enough args the binders we are cancelling with
409         -- the args supplied are, in effect, ocurring inside a lambda.
410         -- So we modify their occurrence info to reflect this fact.
411         -- Example:     (\ x y z -> e) p q
412         --          ==> (\z -> e[p/x, q/y])
413         --      but we should behave as if x and y are marked "inside lambda".
414         -- The occurrence analyser does not mark them so itself because then we
415         -- do badly on the very common case of saturated lambdas applications:
416         --              (\ x y z -> e) p q r
417         --          ==> e[p/x, q/y, r/z]
418         --
419     zapped_binder_args_pairs = [ ((id, markDangerousToDup occ_info), arg)
420                                | ((id, occ_info), arg) <- binder_args_pairs ]
421
422     collect_val_args :: InBinder                -- Binder
423                      -> [OutArg]                -- Arguments
424                      -> ([(InBinder,OutArg)],   -- Binder,arg pairs (ToDo: a maybe?)
425                          [InBinder],            -- Leftover binders (ToDo: a maybe)
426                          [OutArg])              -- Leftover args
427
428         -- collect_val_args strips off the leading ValArgs from
429         -- the current arg list, returning them along with the
430         -- depleted list
431     collect_val_args binder []   = ([], [binder], [])
432     collect_val_args binder (arg : args) | isValArg arg
433         = ([(binder,arg)], [], args)
434
435 #ifdef DEBUG
436     collect_val_args _ (other_val_arg : _) = panic "collect_val_args"
437                 -- TyArg should never meet a Lam
438 #endif
439 \end{code}
440
441
442 Let expressions
443 ~~~~~~~~~~~~~~~
444
445 \begin{code}
446 simplExpr env (Let bind body) args
447   | not (switchIsSet env SimplNoLetFromApp)             -- The common case
448   = simplBind env bind (\env -> simplExpr env body args)
449                        (computeResultType env body args)
450
451   | otherwise           -- No float from application
452   = simplBind env bind (\env -> simplExpr env body [])
453                        (computeResultType env body [])  `thenSmpl` \ let_expr' ->
454     returnSmpl (mkGenApp let_expr' args)
455 \end{code}
456
457 Case expressions
458 ~~~~~~~~~~~~~~~~
459
460 \begin{code}
461 simplExpr env expr@(Case scrut alts) args
462   = simplCase env scrut alts (\env rhs -> simplExpr env rhs args)
463                              (computeResultType env expr args)
464 \end{code}
465
466
467 Set-cost-centre
468 ~~~~~~~~~~~~~~~
469
470 A special case we do:
471 \begin{verbatim}
472         scc "foo" (\x -> e)  ===>   \x -> scc "foo" e
473 \end{verbatim}
474 Simon thinks it's OK, at least for lexical scoping; and it makes
475 interfaces change less (arities).
476
477 \begin{code}
478 simplExpr env (SCC cc (Lam binder body)) args
479   = simplExpr env (Lam binder (SCC cc body)) args
480 \end{code}
481
482 Some other slightly turgid SCC tidying-up cases:
483 \begin{code}
484 simplExpr env (SCC cc1 expr@(SCC _ _)) args
485   = simplExpr env expr args
486     -- the outer _scc_ serves no purpose
487
488 simplExpr env (SCC cc expr) args
489   | squashableDictishCcExpr cc expr
490   = simplExpr env expr args
491     -- the DICT-ish CC is no longer serving any purpose
492 \end{code}
493
494 NB: for other set-cost-centre we move arguments inside the body.
495 ToDo: check with Patrick that this is ok.
496
497 \begin{code}
498 simplExpr env (SCC cost_centre body) args
499   = let
500         new_env = setEnclosingCC env (EnclosingCC cost_centre)
501     in
502     simplExpr new_env body args         `thenSmpl` \ body' ->
503     returnSmpl (SCC cost_centre body')
504 \end{code}
505
506 %************************************************************************
507 %*                                                                      *
508 \subsection{Simplify RHS of a Let/Letrec}
509 %*                                                                      *
510 %************************************************************************
511
512 simplRhsExpr does arity-expansion.  That is, given:
513
514         * a right hand side /\ tyvars -> \a1 ... an -> e
515         * the information (stored in BinderInfo) that the function will always
516           be applied to at least k arguments
517
518 it transforms the rhs to
519
520         /\tyvars -> \a1 ... an b(n+1) ... bk -> (e b(n+1) ... bk)
521
522 This is a Very Good Thing!
523
524 \begin{code}
525 simplRhsExpr
526         :: SimplEnv
527         -> InBinder
528         -> InExpr
529         -> SmplM OutExpr
530
531 simplRhsExpr env binder@(id,occ_info) rhs
532   | dont_eta_expand rhs
533   = simplExpr rhs_env rhs []
534
535   | otherwise   -- Have a go at eta expansion
536   =     -- Deal with the big lambda part
537     mapSmpl cloneTyVarSmpl tyvars                       `thenSmpl` \ tyvars' ->
538     let
539         lam_env  = extendTyEnvList rhs_env (tyvars `zip` (mkTyVarTys tyvars'))
540     in
541         -- Deal with the little lambda part
542         -- Note that we call simplLam even if there are no binders, in case
543         -- it can do arity expansion.
544     simplLam lam_env binders body min_no_of_args        `thenSmpl` \ lambda' ->
545
546         -- Put it back together
547     returnSmpl (
548        (if switchIsSet env SimplDoEtaReduction
549        then mkTyLamTryingEta
550        else mkTyLam) tyvars' lambda'
551     )
552   where
553         -- Note from ANDY:
554         -- If you say {-# INLINE #-} then you get what's coming to you;
555         -- you are saying inline the rhs, please.
556         -- we might want a {-# INLINE UNSIMPLIFIED #-} option.
557     rhs_env | simplIdWantsToBeINLINEd id env = filterUnfoldEnvForInlines env
558             | otherwise                      = env
559
560     (uvars, tyvars, binders, body) = collectBinders rhs
561
562     min_no_of_args | not (null binders)                 &&      -- It's not a thunk
563                      switchIsSet env SimplDoArityExpand         -- Arity expansion on
564                    = getBinderInfoArity occ_info - length binders
565
566                    | otherwise  -- Not a thunk
567                    = 0          -- Play safe!
568
569         -- dont_eta_expand prevents eta expansion in silly situations.
570         -- For example, consider the defn
571         --      x = y
572         -- It would be silly to eta expand the "y", because it would just
573         -- get eta-reduced back to y.  Furthermore, if this was a top level defn,
574         -- and x was exported, then the defn won't be eliminated, so this
575         -- silly expand/reduce cycle will happen every time, which makes the
576         -- simplifier loop!.
577         -- The solution is to not even try eta expansion unless the rhs looks
578         -- non-trivial.
579     dont_eta_expand (Lit _)     = True
580     dont_eta_expand (Var _)     = True
581     dont_eta_expand (Con _ _)   = True
582     dont_eta_expand (App f a)
583       | notValArg    a          = dont_eta_expand f
584     dont_eta_expand (Lam x b)
585       | notValBinder x          = dont_eta_expand b
586     dont_eta_expand _           = False
587 \end{code}
588
589
590 %************************************************************************
591 %*                                                                      *
592 \subsection{Simplify a lambda abstraction}
593 %*                                                                      *
594 %************************************************************************
595
596 Simplify (\binders -> body) trying eta expansion and reduction, given that
597 the abstraction will always be applied to at least min_no_of_args.
598
599 \begin{code}
600 simplLam env binders body min_no_of_args
601   | not (switchIsSet env SimplDoLambdaEtaExpansion) ||  -- Bale out if eta expansion off
602     null potential_extra_binder_tys                 ||  -- or ain't a function
603     no_of_extra_binders == 0                            -- or no extra binders needed
604   = cloneIds env binders                `thenSmpl` \ binders' ->
605     let
606         new_env = extendIdEnvWithClones env binders binders'
607     in
608     simplExpr new_env body []           `thenSmpl` \ body' ->
609     returnSmpl (
610       (if switchIsSet new_env SimplDoEtaReduction
611        then mkValLamTryingEta
612        else mkValLam) binders' body'
613     )
614
615   | otherwise                           -- Eta expansion possible
616   = tick EtaExpansion                   `thenSmpl_`
617     cloneIds env binders                `thenSmpl` \ binders' ->
618     let
619         new_env = extendIdEnvWithClones env binders binders'
620     in
621     newIds extra_binder_tys                             `thenSmpl` \ extra_binders' ->
622     simplExpr new_env body (map VarArg extra_binders')  `thenSmpl` \ body' ->
623     returnSmpl (
624       (if switchIsSet new_env SimplDoEtaReduction
625        then mkValLamTryingEta
626        else mkValLam) (binders' ++ extra_binders') body'
627     )
628
629   where
630     (potential_extra_binder_tys, res_ty)
631         = splitFunTy (simplTy env (coreExprType (unTagBinders body)))
632         -- Note: it's possible that simplLam will be applied to something
633         -- with a forall type.  Eg when being applied to the rhs of
634         --              let x = wurble
635         -- where wurble has a forall-type, but no big lambdas at the top.
636         -- We could be clever an insert new big lambdas, but we don't bother.
637
638     extra_binder_tys = take no_of_extra_binders potential_extra_binder_tys
639
640     no_of_extra_binders =       -- First, use the info about how many args it's
641                                 -- always applied to in its scope
642                            min_no_of_args
643
644                                 -- Next, try seeing if there's a lambda hidden inside
645                                 -- something cheap
646                            `max`
647                            etaExpandCount body
648
649                                 -- Finally, see if it's a state transformer, in which
650                                 -- case we eta-expand on principle! This can waste work,
651                                 -- but usually doesn't
652                            `max`
653                            case potential_extra_binder_tys of
654                                 [ty] | ty `eqTy` realWorldStateTy -> 1
655                                 other                             -> 0
656
657 \end{code}
658
659
660 %************************************************************************
661 %*                                                                      *
662 \subsection[Simplify-let]{Let-expressions}
663 %*                                                                      *
664 %************************************************************************
665
666 \begin{code}
667 simplBind :: SimplEnv
668           -> InBinding
669           -> (SimplEnv -> SmplM OutExpr)
670           -> OutType
671           -> SmplM OutExpr
672 \end{code}
673
674 When floating cases out of lets, remember this:
675
676         let x* = case e of alts
677         in <small expr>
678
679 where x* is sure to be demanded or e is a cheap operation that cannot
680 fail, e.g. unboxed addition.  Here we should be prepared to duplicate
681 <small expr>.  A good example:
682
683         let x* = case y of
684                    p1 -> build e1
685                    p2 -> build e2
686         in
687         foldr c n x*
688 ==>
689         case y of
690           p1 -> foldr c n (build e1)
691           p2 -> foldr c n (build e2)
692
693 NEW: We use the same machinery that we use for case-of-case to
694 *always* do case floating from let, that is we let bind and abstract
695 the original let body, and let the occurrence analyser later decide
696 whether the new let should be inlined or not. The example above
697 becomes:
698
699 ==>
700       let join_body x' = foldr c n x'
701         in case y of
702         p1 -> let x* = build e1
703                 in join_body x*
704         p2 -> let x* = build e2
705                 in join_body x*
706
707 note that join_body is a let-no-escape.
708 In this particular example join_body will later be inlined,
709 achieving the same effect.
710 ToDo: check this is OK with andy
711
712
713
714 \begin{code}
715 -- Dead code is now discarded by the occurrence analyser,
716
717 simplBind env (NonRec binder@(id,occ_info) rhs) body_c body_ty
718   |  inlineUnconditionally ok_to_dup occ_info
719   = body_c (extendIdEnvWithInlining env env binder rhs)
720
721 -- Try let-to-case
722 -- It's important to try let-to-case before floating. Consider
723 --
724 --      let a*::Int = case v of {p1->e1; p2->e2}
725 --      in b
726 --
727 -- (The * means that a is sure to be demanded.)
728 -- If we do case-floating first we get this:
729 --
730 --      let k = \a* -> b
731 --      in case v of
732 --              p1-> let a*=e1 in k a
733 --              p2-> let a*=e2 in k a
734 --
735 -- Now watch what happens if we do let-to-case first:
736 --
737 --      case (case v of {p1->e1; p2->e2}) of
738 --        Int a# -> let a*=I# a# in b
739 -- ===>
740 --      let k = \a# -> let a*=I# a# in b
741 --      in case v of
742 --              p1 -> case e1 of I# a# -> k a#
743 --              p1 -> case e1 of I# a# -> k a#
744 --
745 -- The latter is clearly better.  (Remember the reboxing let-decl
746 -- for a is likely to go away, because after all b is strict in a.)
747
748   | will_be_demanded &&
749     try_let_to_case &&
750     type_ok_for_let_to_case rhs_ty &&
751     not (manifestlyWHNF rhs)
752         -- note: no "manifestlyBottom rhs" in there... (comment below)
753     = tick Let2Case                             `thenSmpl_`
754       mkIdentityAlts rhs_ty                     `thenSmpl` \ id_alts ->
755       simplCase env rhs id_alts (\env rhs -> done_float env rhs body_c) body_ty
756         {-
757         We do not do let to case for WHNFs, e.g.
758
759           let x = a:b in ...
760           =/=>
761           case a:b of x in ...
762
763           as this is less efficient.
764           but we don't mind doing let-to-case for "bottom", as that
765           will
766           allow us to remove more dead code, if anything:
767           let x = error in ...
768           ===>
769           case error  of x -> ...
770           ===>
771           error
772
773           Notice that let to case occurs only if x is used strictly in
774           its body (obviously).
775         -}
776
777   | (will_be_demanded && not no_float) ||
778     always_float_let_from_let ||
779     floatExposesHNF float_lets float_primops ok_to_dup rhs
780   = try_float env rhs body_c
781
782   | otherwise
783   = done_float env rhs body_c
784
785   where
786     will_be_demanded = willBeDemanded (getIdDemandInfo id)
787     rhs_ty           = idType id
788
789     float_lets                = switchIsSet env SimplFloatLetsExposingWHNF
790     float_primops             = switchIsSet env SimplOkToFloatPrimOps
791     ok_to_dup                 = switchIsSet env SimplOkToDupCode
792     always_float_let_from_let = switchIsSet env SimplAlwaysFloatLetsFromLets
793     try_let_to_case           = switchIsSet env SimplLetToCase
794     no_float                  = switchIsSet env SimplNoLetFromStrictLet
795
796     -------------------------------------------
797     done_float env rhs body_c
798         = simplRhsExpr env binder rhs   `thenSmpl` \ rhs' ->
799           completeLet env binder rhs rhs' body_c body_ty
800
801     ---------------------------------------
802     try_float env (Let bind rhs) body_c
803       = tick LetFloatFromLet                    `thenSmpl_`
804         simplBind env (fix_up_demandedness will_be_demanded bind)
805                       (\env -> try_float env rhs body_c) body_ty
806
807     try_float env (Case scrut alts) body_c
808       | will_be_demanded || (float_primops && is_cheap_prim_app scrut)
809       = tick CaseFloatFromLet                           `thenSmpl_`
810
811         -- First, bind large let-body if necessary
812         if no_need_to_bind_large_body then
813             simplCase env scrut alts (\env rhs -> try_float env rhs body_c) body_ty
814         else
815             bindLargeRhs env [binder] body_ty body_c    `thenSmpl` \ (extra_binding, new_body) ->
816             let
817                 body_c' = \env -> simplExpr env new_body []
818             in
819             simplCase env scrut alts
820                       (\env rhs -> try_float env rhs body_c')
821                       body_ty                           `thenSmpl` \ case_expr ->
822
823             returnSmpl (Let extra_binding case_expr)
824       where
825         no_need_to_bind_large_body
826           = ok_to_dup || isSingleton (nonErrorRHSs alts)
827
828     try_float env other_rhs body_c = done_float env other_rhs body_c
829 \end{code}
830
831 Letrec expressions
832 ~~~~~~~~~~~~~~~~~~
833
834 Simplify each RHS, float any let(recs) from the RHSs (if let-floating is
835 on and it'll expose a HNF), and bang the whole resulting mess together
836 into a huge letrec.
837
838 1. Any "macros" should be expanded.  The main application of this
839 macro-expansion is:
840
841         letrec
842                 f = ....g...
843                 g = ....f...
844         in
845         ....f...
846
847 Here we would like the single call to g to be inlined.
848
849 We can spot this easily, because g will be tagged as having just one
850 occurrence.  The "inlineUnconditionally" predicate is just what we want.
851
852 A worry: could this lead to non-termination?  For example:
853
854         letrec
855                 f = ...g...
856                 g = ...f...
857                 h = ...h...
858         in
859         ..h..
860
861 Here, f and g call each other (just once) and neither is used elsewhere.
862 But it's OK:
863
864 * the occurrence analyser will drop any (sub)-group that isn't used at
865   all.
866
867 * If the group is used outside itself (ie in the "in" part), then there
868   can't be a cyle.
869
870 ** IMPORTANT: check that NewOccAnal has the property that a group of
871    bindings like the above has f&g dropped.! ***
872
873
874 2. We'd also like to pull out any top-level let(rec)s from the
875 rhs of the defns:
876
877         letrec
878                 f = let h = ... in \x -> ....h...f...h...
879         in
880         ...f...
881 ====>
882         letrec
883                 h = ...
884                 f = \x -> ....h...f...h...
885         in
886         ...f...
887
888 But floating cases is less easy?  (Don't for now; ToDo?)
889
890
891 3.  We'd like to arrange that the RHSs "know" about members of the
892 group that are bound to constructors.  For example:
893
894     let rec
895        d.Eq      = (==,/=)
896        f a b c d = case d.Eq of (h,_) -> let x = (a,b); y = (c,d) in not (h x y)
897        /= a b    = unpack tuple a, unpack tuple b, call f
898     in d.Eq
899
900 here, by knowing about d.Eq in f's rhs, one could get rid of
901 the case (and break out the recursion completely).
902 [This occurred with more aggressive inlining threshold (4),
903 nofib/spectral/knights]
904
905 How to do it?
906         1: we simplify constructor rhss first.
907         2: we record the "known constructors" in the environment
908         3: we simplify the other rhss, with the knowledge about the constructors
909
910
911
912 \begin{code}
913 simplBind env (Rec pairs) body_c body_ty
914   =     -- Do floating, if necessary
915     (if float_lets || always_float_let_from_let
916      then
917         mapSmpl float pairs     `thenSmpl` \ floated_pairs_s ->
918         returnSmpl (concat floated_pairs_s)
919      else
920         returnSmpl pairs
921     )                                   `thenSmpl` \ floated_pairs ->
922     let
923         binders = map fst floated_pairs
924     in
925     cloneIds env binders                `thenSmpl` \ ids' ->
926     let
927         env_w_clones = extendIdEnvWithClones env binders ids'
928         triples      = ids' `zip` floated_pairs
929     in
930
931     simplRecursiveGroup env_w_clones triples    `thenSmpl` \ (binding, new_env) ->
932
933     body_c new_env                              `thenSmpl` \ body' ->
934
935     returnSmpl (Let binding body')
936
937   where
938     ------------ Floating stuff -------------------
939
940     float_lets                = switchIsSet env SimplFloatLetsExposingWHNF
941     always_float_let_from_let = switchIsSet env SimplAlwaysFloatLetsFromLets
942
943     float (binder,rhs)
944       = let
945             pairs_s = float_pair (binder,rhs)
946         in
947         case pairs_s of
948           [_] -> returnSmpl pairs_s
949           more_than_one
950             -> tickN LetFloatFromLet (length pairs_s - 1) `thenSmpl_`
951                 -- It's important to increment the tick counts if we
952                 -- do any floating.  A situation where this turns out
953                 -- to be important is this:
954                 -- Float in produces:
955                 --      letrec  x = let y = Ey in Ex
956                 --      in B
957                 -- Now floating gives this:
958                 --      letrec x = Ex
959                 --             y = Ey
960                 --      in B
961                 --- We now want to iterate once more in case Ey doesn't
962                 -- mention x, in which case the y binding can be pulled
963                 -- out as an enclosing let(rec), which in turn gives
964                 -- the strictness analyser more chance.
965                 returnSmpl pairs_s
966
967     float_pairs pairs = concat (map float_pair pairs)
968
969     float_pair (binder, rhs)
970         | always_float_let_from_let ||
971           floatExposesHNF True False False rhs
972         = (binder,rhs') : pairs'
973
974         | otherwise
975         = [(binder,rhs)]
976         where
977           (pairs', rhs') = do_float rhs
978
979         -- Float just pulls out any top-level let(rec) bindings
980     do_float :: InExpr -> ([(InBinder,InExpr)], InExpr)
981     do_float (Let (Rec pairs) body)     = (float_pairs pairs    ++ pairs', body')
982                                             where
983                                               (pairs', body') = do_float body
984     do_float (Let (NonRec id rhs) body) = (float_pair (id,rhs) ++ pairs', body')
985                                             where
986                                               (pairs', body') = do_float body
987     do_float other                          = ([], other)
988
989 simplRecursiveGroup env triples
990   =     -- Toss out all the dead pairs?  No, there shouldn't be any!
991         -- Dead code is discarded by the occurrence analyser
992     let
993             -- Separate the live triples into "inline"able and
994             -- "ordinary" We're paranoid about duplication!
995         (inline_triples, ordinary_triples)
996           = partition is_inline_triple triples
997
998         is_inline_triple (_, ((_,occ_info),_))
999           = inlineUnconditionally False {-not ok_to_dup-} occ_info
1000
1001             -- Now add in the inline_pairs info (using "env_w_clones"),
1002             -- so that we will save away suitably-clone-laden envs
1003             -- inside the InlineIts...).
1004
1005             -- NOTE ALSO that we tie a knot here, because the
1006             -- saved-away envs must also include these very inlinings
1007             -- (they aren't stored anywhere else, and a late one might
1008             -- be used in an early one).
1009
1010         env_w_inlinings = foldl add_inline env inline_triples
1011
1012         add_inline env (id', (binder,rhs))
1013           = extendIdEnvWithInlining env env_w_inlinings binder rhs
1014
1015             -- Separate the remaining bindings into the ones which
1016             -- need to be dealt with first (the "early" ones)
1017             -- and the others (the "late" ones)
1018         (early_triples, late_triples)
1019           = partition is_early_triple ordinary_triples
1020
1021         is_early_triple (_, (_, Con _ _)) = True
1022         is_early_triple (i, _           ) = idWantsToBeINLINEd i
1023     in
1024         -- Process the early bindings first
1025     mapSmpl (do_one_binding env_w_inlinings) early_triples      `thenSmpl` \ early_triples' ->
1026
1027         -- Now further extend the environment to record our knowledge
1028         -- about the form of the binders bound in the constructor bindings
1029     let
1030         env_w_early_info = foldr add_early_info env_w_inlinings early_triples'
1031         add_early_info (binder, (id', rhs')) env = extendUnfoldEnvGivenRhs env binder id' rhs'
1032     in
1033         -- Now process the non-constructor bindings
1034     mapSmpl (do_one_binding env_w_early_info) late_triples      `thenSmpl` \ late_triples' ->
1035
1036         -- Phew! We're done
1037     let
1038         binding = Rec (map snd early_triples' ++ map snd late_triples')
1039     in
1040     returnSmpl (binding, env_w_early_info)
1041   where
1042
1043     do_one_binding env (id', (binder,rhs))
1044       = simplRhsExpr env binder rhs `thenSmpl` \ rhs' ->
1045         returnSmpl (binder, (id', rhs'))
1046 \end{code}
1047
1048
1049 @completeLet@ looks at the simplified post-floating RHS of the
1050 let-expression, and decides what to do.  There's one interesting
1051 aspect to this, namely constructor reuse.  Consider
1052 @
1053         f = \x -> case x of
1054                     (y:ys) -> y:ys
1055                     []     -> ...
1056 @
1057 Is it a good idea to replace the rhs @y:ys@ with @x@?  This depends a
1058 bit on the compiler technology, but in general I believe not. For
1059 example, here's some code from a real program:
1060 @
1061 const.Int.max.wrk{-s2516-} =
1062     \ upk.s3297#  upk.s3298# ->
1063         let {
1064           a.s3299 :: Int
1065           _N_ {-# U(P) #-}
1066           a.s3299 = I#! upk.s3297#
1067         } in
1068           case (const.Int._tagCmp.wrk{-s2513-} upk.s3297# upk.s3298#) of {
1069             _LT -> I#! upk.s3298#
1070             _EQ -> a.s3299
1071             _GT -> a.s3299
1072           }
1073 @
1074 The a.s3299 really isn't doing much good.  We'd be better off inlining
1075 it.  (Actually, let-no-escapery means it isn't as bad as it looks.)
1076
1077 So the current strategy is to inline all known-form constructors, and
1078 only do the reverse (turn a constructor application back into a
1079 variable) when we find a let-expression:
1080 @
1081         let x = C a1 .. an
1082         in
1083         ... (let y = C a1 .. an in ...) ...
1084 @
1085 where it is always good to ditch the binding for y, and replace y by
1086 x.  That's just what completeLetBinding does.
1087
1088 \begin{code}
1089 completeLet
1090         :: SimplEnv
1091         -> InBinder
1092         -> InExpr               -- Original RHS
1093         -> OutExpr              -- The simplified RHS
1094         -> (SimplEnv -> SmplM OutExpr)          -- Body handler
1095         -> OutType              -- Type of body
1096         -> SmplM OutExpr
1097
1098 completeLet env binder@(id,binder_info) old_rhs new_rhs body_c body_ty
1099
1100   -- See if RHS is an atom, or a reusable constructor
1101   | maybeToBool maybe_atomic_rhs
1102   = let
1103         new_env = extendIdEnvWithAtom env binder rhs_atom
1104     in
1105     tick atom_tick_type                 `thenSmpl_`
1106     body_c new_env
1107
1108   -- Maybe the rhs is an application of error, and sure to be demanded
1109   | will_be_demanded &&
1110     maybeToBool maybe_error_app
1111   = tick CaseOfError                    `thenSmpl_`
1112     returnSmpl retyped_error_app
1113
1114   -- The general case
1115   | otherwise
1116   = cloneId env binder                  `thenSmpl` \ id' ->
1117     let
1118         env1    = extendIdEnvWithClone env binder id'
1119         new_env = extendUnfoldEnvGivenRhs env1 binder id' new_rhs
1120     in
1121     body_c new_env                      `thenSmpl` \ body' ->
1122     returnSmpl (Let (NonRec id' new_rhs) body')
1123
1124   where
1125     will_be_demanded = willBeDemanded (getIdDemandInfo id)
1126     try_to_reuse_constr   = switchIsSet env SimplReuseCon
1127
1128     Just (rhs_atom, atom_tick_type) = maybe_atomic_rhs
1129
1130     maybe_atomic_rhs :: Maybe (OutArg, TickType)
1131         -- If the RHS is atomic, we return Just (atom, tick type)
1132         -- otherwise Nothing
1133
1134     maybe_atomic_rhs
1135       = case new_rhs of
1136           Var var -> Just (VarArg var, AtomicRhs)
1137
1138           Lit lit | not (isNoRepLit lit)
1139             -> Just (LitArg lit, AtomicRhs)
1140
1141           Con con con_args
1142             | try_to_reuse_constr
1143                    -- Look out for
1144                    --   let v = C args
1145                    --   in
1146                    --- ...(let w = C same-args in ...)...
1147                    -- Then use v instead of w.   This may save
1148                    -- re-constructing an existing constructor.
1149              -> case (lookForConstructor env con con_args) of
1150                   Nothing  -> Nothing
1151                   Just var -> Just (VarArg var, ConReused)
1152
1153           other -> Nothing
1154
1155     maybe_error_app        = maybeErrorApp new_rhs (Just body_ty)
1156     Just retyped_error_app = maybe_error_app
1157 \end{code}
1158
1159 %************************************************************************
1160 %*                                                                      *
1161 \subsection[Simplify-atoms]{Simplifying atoms}
1162 %*                                                                      *
1163 %************************************************************************
1164
1165 \begin{code}
1166 simplArg :: SimplEnv -> InArg -> OutArg
1167
1168 simplArg env (LitArg lit) = LitArg lit
1169 simplArg env (TyArg  ty)  = TyArg  (simplTy env ty)
1170
1171 simplArg env (VarArg id)
1172   | isLocallyDefined id
1173   = case lookupId env id of
1174         Just (ItsAnAtom atom) -> atom
1175         Just (InlineIt _ _ _) -> pprPanic "simplArg InLineIt:" (ppAbove (ppr PprDebug id) (pprSimplEnv env))
1176         Nothing               -> VarArg id      -- Must be an uncloned thing
1177
1178   | otherwise
1179   =     -- Not locally defined, so no change
1180     VarArg id
1181 \end{code}
1182
1183
1184 %************************************************************************
1185 %*                                                                      *
1186 \subsection[Simplify-quickies]{Some local help functions}
1187 %*                                                                      *
1188 %************************************************************************
1189
1190
1191 \begin{code}
1192 -- fix_up_demandedness switches off the willBeDemanded Info field
1193 -- for bindings floated out of a non-demanded let
1194 fix_up_demandedness True {- Will be demanded -} bind
1195    = bind       -- Simple; no change to demand info needed
1196 fix_up_demandedness False {- May not be demanded -} (NonRec binder rhs)
1197    = NonRec (un_demandify binder) rhs
1198 fix_up_demandedness False {- May not be demanded -} (Rec pairs)
1199    = Rec [(un_demandify binder, rhs) | (binder,rhs) <- pairs]
1200
1201 un_demandify (id, occ_info) = (id `addIdDemandInfo` noInfo, occ_info)
1202
1203 is_cheap_prim_app (Prim op _) = primOpOkForSpeculation op
1204 is_cheap_prim_app other       = False
1205
1206 computeResultType :: SimplEnv -> InExpr -> [OutArg] -> OutType
1207 computeResultType env expr args
1208   = go expr_ty' args
1209   where
1210     expr_ty  = coreExprType (unTagBinders expr)
1211     expr_ty' = simplTy env expr_ty
1212
1213     go ty [] = ty
1214     go ty (TyArg ty_arg : args) = go (mkAppTy ty ty_arg) args
1215     go ty (a:args) | isValArg a = case (getFunTy_maybe ty) of
1216                                     Just (_, res_ty) -> go res_ty args
1217                                     Nothing          -> panic "computeResultType"
1218 \end{code}
1219