[project @ 2002-01-25 10:28:12 by simonmar]
[ghc-hetmet.git] / ghc / compiler / ghci / ByteCodeGen.lhs
index 852b79b..2e3a9e8 100644 (file)
@@ -18,50 +18,52 @@ import Id           ( Id, idType, isDataConId_maybe, isPrimOpId_maybe, isFCallId,
 import ForeignCall     ( ForeignCall(..), CCallTarget(..), CCallSpec(..) )
 import OrdList         ( OrdList, consOL, snocOL, appOL, unitOL, 
                          nilOL, toOL, concatOL, fromOL )
-import FiniteMap       ( FiniteMap, addListToFM, listToFM,
+import FiniteMap       ( FiniteMap, addListToFM, listToFM, elemFM,
                          addToFM, lookupFM, fmToList )
 import CoreSyn
 import PprCore         ( pprCoreExpr )
 import Literal         ( Literal(..), literalPrimRep )
 import PrimRep         ( PrimRep(..) )
 import PrimOp          ( PrimOp(..) )
-import CStrings                ( CLabelString )
 import CoreFVs         ( freeVars )
-import Type            ( typePrimRep, splitTyConApp_maybe, isTyVarTy, splitForAllTys )
+import Type            ( typePrimRep, splitTyConApp_maybe, isTyVarTy )
 import DataCon         ( dataConTag, fIRST_TAG, dataConTyCon, 
                           dataConWrapId, isUnboxedTupleCon )
 import TyCon           ( TyCon(..), tyConFamilySize, isDataTyCon, tyConDataCons,
                          isFunTyCon, isUnboxedTupleTyCon )
 import Class           ( Class, classTyCon )
 import Type            ( Type, repType, splitRepFunTys )
-import Util            ( zipEqual, zipWith4Equal, naturalMergeSortLe, nOfThem )
+import Util            ( zipEqual, zipWith4Equal, naturalMergeSortLe, nOfThem,
+                         isSingleton, lengthIs )
 import Var             ( isTyVar )
 import VarSet          ( VarSet, varSetElems )
-import PrimRep         ( getPrimRepSize, isFollowableRep )
+import PrimRep         ( isFollowableRep )
 import CmdLineOpts     ( DynFlags, DynFlag(..) )
 import ErrUtils                ( showPass, dumpIfSet_dyn )
 import Unique          ( mkPseudoUnique3 )
 import FastString      ( FastString(..) )
 import Panic           ( GhcException(..) )
 import PprType         ( pprType )
+import SMRep           ( arrWordsHdrSize, arrPtrsHdrSize )
+import Constants       ( wORD_SIZE )
 import ByteCodeInstr   ( BCInstr(..), ProtoBCO(..), nameOfProtoBCO, bciStackUse )
 import ByteCodeItbls   ( ItblEnv, mkITbls )
 import ByteCodeLink    ( UnlinkedBCO, UnlinkedBCOExpr, assembleBCO,
-                         ClosureEnv, HValue, filterNameMap,
+                         ClosureEnv, HValue, filterNameMap, linkFail,
                          iNTERP_STACK_CHECK_THRESH )
-import ByteCodeFFI     ( taggedSizeW, untaggedSizeW, mkMarshalCode )
+import ByteCodeFFI     ( taggedSizeW, untaggedSizeW, mkMarshalCode, moan64 )
 import Linker          ( lookupSymbol )
 
 import List            ( intersperse, sortBy, zip4 )
 import Foreign         ( Ptr(..), mallocBytes )
-import Addr            ( Addr(..), nullAddr, addrToInt, writeCharOffAddr )
+import Addr            ( Addr(..), writeCharOffAddr )
 import CTypes          ( CInt )
 import Exception       ( throwDyn )
 
 import PrelBase                ( Int(..) )
 import PrelGHC         ( ByteArray# )
-import IOExts          ( unsafePerformIO )
 import PrelIOBase      ( IO(..) )
+import Monad           ( when )
 
 \end{code}
 
@@ -85,10 +87,15 @@ byteCodeGen dflags binds local_tycons local_classes
         let flatBinds = concatMap getBind binds
             getBind (NonRec bndr rhs) = [(bndr, freeVars rhs)]
             getBind (Rec binds)       = [(bndr, freeVars rhs) | (bndr,rhs) <- binds]
-            final_state = runBc (BcM_State [] 0) 
-                                (mapBc (schemeR True) flatBinds
-                                       `thenBc_` returnBc ())
-            (BcM_State proto_bcos final_ctr) = final_state
+
+        (BcM_State proto_bcos final_ctr mallocd, ())
+           <- runBc (BcM_State [] 0 []) 
+                    (mapBc (schemeR True []) flatBinds `thenBc_` returnBc ())
+                       --               ^^
+                       -- better be no free vars in these top-level bindings
+
+        when (not (null mallocd))
+             (panic "ByteCodeGen.byteCodeGen: missing final emitBc?")
 
         dumpIfSet_dyn dflags Opt_D_dump_BCOs
            "Proto-bcos" (vcat (intersperse (char ' ') (map ppr proto_bcos)))
@@ -112,9 +119,16 @@ coreExprToBCOs dflags expr
                                     (panic "invented_id's type")
       let invented_name = idName invented_id
 
-      let (BcM_State all_proto_bcos final_ctr) 
-             = runBc (BcM_State [] 0) 
-                     (schemeR True (invented_id, freeVars expr))
+         annexpr = freeVars expr
+         fvs = filter (not.isTyVar) (varSetElems (fst annexpr))
+
+      (BcM_State all_proto_bcos final_ctr mallocd, ()) 
+         <- runBc (BcM_State [] 0 []) 
+                  (schemeR True fvs (invented_id, annexpr))
+
+      when (not (null mallocd))
+           (panic "ByteCodeGen.coreExprToBCOs: missing final emitBc?")
+
       dumpIfSet_dyn dflags Opt_D_dump_BCOs
          "Proto-bcos" (vcat (intersperse (char ' ') (map ppr all_proto_bcos)))
 
@@ -157,8 +171,8 @@ ppBCEnv p
 
 -- Create a BCO and do a spot of peephole optimisation on the insns
 -- at the same time.
-mkProtoBCO nm instrs_ordlist origin
-   = ProtoBCO nm maybe_with_stack_check origin
+mkProtoBCO nm instrs_ordlist origin mallocd_blocks
+   = ProtoBCO nm maybe_with_stack_check origin mallocd_blocks
      where
         -- Overestimate the stack usage (in words) of this BCO,
         -- and if >= iNTERP_STACK_CHECK_THRESH, add an explicit
@@ -198,8 +212,8 @@ mkProtoBCO nm instrs_ordlist origin
 -- variable to which this value was bound, so as to give the
 -- resulting BCO a name.  Bool indicates top-levelness.
 
-schemeR :: Bool -> (Id, AnnExpr Id VarSet) -> BcM ()
-schemeR is_top (nm, rhs) 
+schemeR :: Bool -> [Id] -> (Id, AnnExpr Id VarSet) -> BcM ()
+schemeR is_top fvs (nm, rhs) 
 {-
    | trace (showSDoc (
               (char ' '
@@ -210,7 +224,7 @@ schemeR is_top (nm, rhs)
    = undefined
 -}
    | otherwise
-   = schemeR_wrk is_top rhs nm (collect [] rhs)
+   = schemeR_wrk is_top fvs rhs nm (collect [] rhs)
 
 
 collect xs (_, AnnNote note e)
@@ -220,7 +234,7 @@ collect xs (_, AnnLam x e)
 collect xs not_lambda
    = (reverse xs, not_lambda)
 
-schemeR_wrk is_top original_body nm (args, body)
+schemeR_wrk is_top fvs original_body nm (args, body)
    | Just dcon <- maybe_toplevel_null_con_rhs
    = --trace ("nullary constructor! " ++ showSDocDebug (ppr nm)) (
      emitBc (mkProtoBCO (getName nm) (toOL [PACK dcon 0, ENTER])
@@ -228,8 +242,7 @@ schemeR_wrk is_top original_body nm (args, body)
      --)
 
    | otherwise
-   = let fvs       = filter (not.isTyVar) (varSetElems (fst original_body))
-         all_args  = reverse args ++ fvs
+   = let all_args  = reverse args ++ fvs
          szsw_args = map taggedIdSizeW all_args
          szw_args  = sum szsw_args
          p_init    = listToFM (zip all_args (mkStackOffsets 0 szsw_args))
@@ -242,7 +255,7 @@ schemeR_wrk is_top original_body nm (args, body)
      where
         maybe_toplevel_null_con_rhs
            | is_top && null args
-           = case snd body of
+           = case nukeTyArgs (snd body) of
                 AnnVar v_wrk 
                    -> case isDataConId_maybe v_wrk of
                          Nothing -> Nothing
@@ -254,6 +267,10 @@ schemeR_wrk is_top original_body nm (args, body)
            | otherwise
            = Nothing
 
+        nukeTyArgs (AnnApp f (_, AnnType _)) = nukeTyArgs (snd f)
+        nukeTyArgs other                     = other
+
+
 -- Let szsw be the sizes in words of some items pushed onto the stack,
 -- which has initial depth d'.  Return the values which the stack environment
 -- should map these items to.
@@ -276,16 +293,16 @@ schemeE d s p e@(fvs, AnnVar v)
 
    | otherwise
    = -- returning an unboxed value.  Heave it on the stack, SLIDE, and RETURN.
-     let (push, szw) = pushAtom True d p (AnnVar v)
-     in  returnBc (push                        -- value onto stack
-                   `appOL`  mkSLIDE szw (d-s)  -- clear to sequel
-                   `snocOL` RETURN v_rep)      -- go
+     pushAtom True d p (AnnVar v)      `thenBc` \ (push, szw) ->
+     returnBc (push                    -- value onto stack
+               `appOL`  mkSLIDE szw (d-s)      -- clear to sequel
+               `snocOL` RETURN v_rep)  -- go
    where
       v_rep = typePrimRep (idType v)
 
 schemeE d s p (fvs, AnnLit literal)
-   = let (push, szw) = pushAtom True d p (AnnLit literal)
-         l_rep = literalPrimRep literal
+   = pushAtom True d p (AnnLit literal)        `thenBc` \ (push, szw) ->
+     let l_rep = literalPrimRep literal
      in  returnBc (push                        -- value onto stack
                    `appOL`  mkSLIDE szw (d-s)  -- clear to sequel
                    `snocOL` RETURN l_rep)      -- go
@@ -294,7 +311,9 @@ schemeE d s p (fvs, AnnLet binds b)
    = let (xs,rhss) = case binds of AnnNonRec x rhs  -> ([x],[rhs])
                                    AnnRec xs_n_rhss -> unzip xs_n_rhss
          n     = length xs
-         fvss  = map (filter (not.isTyVar).varSetElems.fst) rhss
+
+        is_local id = not (isTyVar id) && elemFM id p'
+         fvss  = map (filter is_local . varSetElems . fst) rhss
 
          -- Sizes of tagged free vars, + 1 for the fn
          sizes = map (\rhs_fvs -> 1 + sum (map taggedIdSizeW rhs_fvs)) fvss
@@ -312,19 +331,27 @@ schemeE d s p (fvs, AnnLet binds b)
 
          -- ToDo: don't build thunks for things with no free variables
          buildThunk dd ([], size, id, off)
-            = PUSH_G (Left (getName id))
-              `consOL` unitOL (MKAP (off+size-1) size)
+            = returnBc (PUSH_G (Left (getName id))
+                        `consOL` unitOL (MKAP (off+size-1) size))
          buildThunk dd ((fv:fvs), size, id, off)
-            = case pushAtom True dd p' (AnnVar fv) of
-                 (push_code, pushed_szw)
-                    -> push_code `appOL`
-                       buildThunk (dd+pushed_szw) (fvs, size, id, off)
+            = pushAtom True dd p' (AnnVar fv) 
+                                       `thenBc` \ (push_code, pushed_szw) ->
+              buildThunk (dd+pushed_szw) (fvs, size, id, off)
+                                       `thenBc` \ more_push_code ->
+              returnBc (push_code `appOL` more_push_code)
+
+         genThunkCode = mapBc (buildThunk d') infos    `thenBc` \ tcodes ->
+                        returnBc (concatOL tcodes)
 
-         thunkCode = concatOL (map (buildThunk d') infos)
          allocCode = toOL (map ALLOC sizes)
+
+        schemeRs [] _ _ = returnBc ()
+        schemeRs (fvs:fvss) (x:xs) (rhs:rhss) = 
+               schemeR False fvs (x,rhs) `thenBc_` schemeRs fvss xs rhss
      in
      schemeE d' s p' b                                 `thenBc`  \ bodyCode ->
-     mapBc (schemeR False) (zip xs rhss)               `thenBc_`
+     schemeRs fvss xs rhss                             `thenBc_`
+     genThunkCode                                      `thenBc` \ thunkCode ->
      returnBc (allocCode `appOL` thunkCode `appOL` bodyCode)
 
 
@@ -357,7 +384,6 @@ schemeE d s p (fvs_case, AnnCase (fvs_scrut, scrut) bndr
      in  trace ("WARNING: ignoring polymorphic case in interpreted mode.\n" ++
                 "   Possibly due to strict polymorphic/functional constructor args.\n" ++
                 "   Your program may leak space unexpectedly.\n")
-                -- ++ showSDoc (char ' ' $$ pprCoreExpr (deAnnotate new_expr) $$ char ' '))
          (schemeE d s p new_expr)
 
 
@@ -481,11 +507,13 @@ schemeE d s p other
 --     (the VoidRep takes up zero stack space).  Also, spot
 --     (# b #) and treat it as  b.
 --
--- 3.  Application of a non-nullary constructor, by defn saturated.
+-- 3.  The fn denotes a ccall.  Defer to generateCCall.
+--
+-- 4.  Application of a non-nullary constructor, by defn saturated.
 --     Split the args into ptrs and non-ptrs, and push the nonptrs, 
 --     then the ptrs, and then do PACK and RETURN.
 --
--- 4.  Otherwise, it must be a function call.  Push the args
+-- 5.  Otherwise, it must be a function call.  Push the args
 --     right to left, SLIDE and ENTER.
 
 schemeT :: Int                 -- Stack depth
@@ -495,45 +523,50 @@ schemeT :: Int            -- Stack depth
         -> BcM BCInstrList
 
 schemeT d s p app
+
 --   | trace ("schemeT: env in = \n" ++ showSDocDebug (ppBCEnv p)) False
 --   = panic "schemeT ?!?!"
 
 --   | trace ("\nschemeT\n" ++ showSDoc (pprCoreExpr (deAnnotate app)) ++ "\n") False
 --   = error "?!?!" 
 
-   -- Handle case 0
+   -- Case 0
    | Just (arg, constr_names) <- maybe_is_tagToEnum_call
-   = pushAtom True d p arg             `bind` \ (push, arg_words) ->
+   = pushAtom True d p arg             `thenBc` \ (push, arg_words) ->
      implement_tagToId constr_names    `thenBc` \ tagToId_sequence ->
      returnBc (push `appOL`  tagToId_sequence            
                     `appOL`  mkSLIDE 1 (d+arg_words-s)
                     `snocOL` ENTER)
 
-   -- Handle case 1
+   -- Case 1
    | is_con_call && null args_r_to_l
    = returnBc (
         (PUSH_G (Left (getName con)) `consOL` mkSLIDE 1 (d-s))
         `snocOL` ENTER
      )
 
-   -- Handle case 2
+   -- Case 2
    | let isVoidRepAtom (_, AnnVar v)    = VoidRep == typePrimRep (idType v)
          isVoidRepAtom (_, AnnNote n e) = isVoidRepAtom e
      in  is_con_call && isUnboxedTupleCon con 
-         && ( (length args_r_to_l == 2 && isVoidRepAtom (last (args_r_to_l)))
-              || (length args_r_to_l == 1)
+         && ( (args_r_to_l `lengthIs` 2 && isVoidRepAtom (last (args_r_to_l)))
+              || (isSingleton args_r_to_l)
             )
-   = --trace (if length args_r_to_l == 1
+   = --trace (if isSingleton args_r_to_l
      --       then "schemeT: unboxed singleton"
      --       else "schemeT: unboxed pair with Void first component") (
      schemeT d s p (head args_r_to_l)
      --)
 
-   -- Cases 3 and 4
+   -- Case 3
+   | Just (CCall ccall_spec) <- isFCallId_maybe fn
+   = generateCCall d s p ccall_spec fn args_r_to_l
+
+   -- Cases 4 and 5
    | otherwise
    = if   is_con_call && isUnboxedTupleCon con
-     then returnBc unboxedTupleException
-     else code `seq` returnBc code
+     then unboxedTupleException
+     else do_pushery d (map snd args_final_r_to_l)
 
    where
       -- Detect and extract relevant info for the tagToEnum kludge.
@@ -542,7 +575,7 @@ schemeT d s p app
                   = case splitTyConApp_maybe (repType ty) of
                        (Just (tyc, [])) |  isDataTyCon tyc
                                         -> map getName (tyConDataCons tyc)
-                       other            -> panic "maybe_is_tagToEnum_call.extract_constr_Ids"
+                       other -> panic "maybe_is_tagToEnum_call.extract_constr_Ids"
            in 
            case app of
               (_, AnnApp (_, AnnApp (_, AnnVar v) (_, AnnType t)) arg)
@@ -579,47 +612,126 @@ schemeT d s p app
            where isPtr = isFollowableRep . atomRep
 
       -- make code to push the args and then do the SLIDE-ENTER thing
-      code          = do_pushery d (map snd args_final_r_to_l)
       tag_when_push = not is_con_call
       narg_words    = sum (map (get_arg_szw . atomRep . snd) args_r_to_l)
       get_arg_szw   = if tag_when_push then taggedSizeW else untaggedSizeW
 
       do_pushery d (arg:args)
-         = let (push, arg_words) = pushAtom tag_when_push d p arg
-           in  push `appOL` do_pushery (d+arg_words) args
+         = pushAtom tag_when_push d p arg      `thenBc` \ (push, arg_words) ->
+           do_pushery (d+arg_words) args       `thenBc` \ more_push_code ->
+           returnBc (push `appOL` more_push_code)
       do_pushery d []
-
-         -- CCALL !
          | Just (CCall ccall_spec) <- isFCallId_maybe fn
-         = generateCCall d s fn ccall_spec
-
+         = panic "schemeT.do_pushery: unexpected ccall"
          | otherwise
          = case maybe_dcon of
-              Just con -> PACK con narg_words `consOL` (
-                          mkSLIDE 1 (d - narg_words - s) `snocOL` ENTER)
+              Just con -> returnBc (
+                             (PACK con narg_words `consOL`
+                              mkSLIDE 1 (d - narg_words - s)) `snocOL`
+                              ENTER
+                          )
               Nothing
-                 -> let (push, arg_words) = pushAtom True d p (AnnVar fn)
-                    in  push 
-                        `appOL` mkSLIDE (narg_words+arg_words) 
-                                        (d - s - narg_words)
-                        `snocOL` ENTER
+                 -> pushAtom True d p (AnnVar fn)      
+                                               `thenBc` \ (push, arg_words) ->
+                    returnBc (push `appOL` mkSLIDE (narg_words+arg_words) 
+                                                   (d - s - narg_words)
+                              `snocOL` ENTER)
 
 
 
-{- Given that the args for a CCall have been pushed onto the Haskell
-   stack, generate the marshalling (machine) code for the ccall, and
-   create bytecodes to call that and then return in the right way.  
+{- Deal with a CCall.  Taggedly push the args onto the stack R->L,
+   deferencing ForeignObj#s and (ToDo: adjusting addrs to point to
+   payloads in Ptr/Byte arrays).  Then, generate the marshalling
+   (machine) code for the ccall, and create bytecodes to call that and
+   then return in the right way.  
 -}
 generateCCall :: Int -> Sequel                 -- stack and sequel depths
-              -> Id                    -- of target, for type info
+              -> BCEnv
               -> CCallSpec             -- where to call
-              -> BCInstrList
+              -> Id                    -- of target, for type info
+              -> [AnnExpr Id VarSet]   -- args (atoms)
+              -> BcM BCInstrList
+
+generateCCall d0 s p ccall_spec@(CCallSpec target cconv safety) fn args_r_to_l
+   = let 
+         -- useful constants
+         addr_usizeW = untaggedSizeW AddrRep
+         addr_tsizeW = taggedSizeW AddrRep
+
+         -- Get the args on the stack, with tags and suitably
+         -- dereferenced for the CCall.  For each arg, return the
+         -- depth to the first word of the bits for that arg, and the
+         -- PrimRep of what was actually pushed.
+
+         pargs d [] = returnBc []
+         pargs d ((_,a):az) 
+            = let rep_arg = atomRep a
+              in case rep_arg of
+                    -- Don't push the FO; instead push the Addr# it
+                    -- contains.
+                    ForeignObjRep
+                       -> pushAtom False{-irrelevant-} d p a
+                                                       `thenBc` \ (push_fo, _) ->
+                          let foro_szW = taggedSizeW ForeignObjRep
+                              d_now    = d + addr_tsizeW
+                              code     = push_fo `appOL` toOL [
+                                            UPK_TAG addr_usizeW 0 0,
+                                            SLIDE addr_tsizeW foro_szW
+                                         ]
+                          in  pargs d_now az           `thenBc` \ rest ->
+                              returnBc ((code, AddrRep) : rest)
+
+                    ArrayRep
+                       -> pargs (d + addr_tsizeW) az   `thenBc` \ rest ->
+                          parg_ArrayishRep arrPtrsHdrSize d p a
+                                                       `thenBc` \ code ->
+                          returnBc ((code,AddrRep):rest)
+
+                    ByteArrayRep
+                       -> pargs (d + addr_tsizeW) az   `thenBc` \ rest ->
+                          parg_ArrayishRep arrWordsHdrSize d p a
+                                                       `thenBc` \ code ->
+                          returnBc ((code,AddrRep):rest)
+
+                    -- Default case: push taggedly, but otherwise intact.
+                    other
+                       -> pushAtom True d p a          `thenBc` \ (code_a, sz_a) ->
+                          pargs (d+sz_a) az            `thenBc` \ rest ->
+                          returnBc ((code_a, rep_arg) : rest)
+
+         -- Do magic for Ptr/Byte arrays.  Push a ptr to the array on
+         -- the stack but then advance it over the headers, so as to
+         -- point to the payload.
+         parg_ArrayishRep hdrSizeW d p a
+            = pushAtom False{-irrel-} d p a `thenBc` \ (push_fo, _) ->
+              -- The ptr points at the header.  Advance it over the
+              -- header and then pretend this is an Addr# (push a tag).
+              returnBc (push_fo `snocOL` 
+                        SWIZZLE 0 (hdrSizeW * untaggedSizeW PtrRep
+                                            * wORD_SIZE) 
+                        `snocOL`
+                        PUSH_TAG addr_usizeW)
 
-generateCCall d s fn ccall_spec@(CCallSpec target cconv safety)
-   = let -- Get the arg and result reps.
-         (a_reps_RAW, maybe_r_rep) = getCCallPrimReps (idType fn)               
+     in
+         pargs d0 args_r_to_l                          `thenBc` \ code_n_reps ->
+     let
+         (pushs_arg, a_reps_pushed_r_to_l) = unzip code_n_reps
+
+         push_args    = concatOL pushs_arg
+         d_after_args = d0 + sum (map taggedSizeW a_reps_pushed_r_to_l)
+         a_reps_pushed_RAW
+            | null a_reps_pushed_r_to_l || head a_reps_pushed_r_to_l /= VoidRep
+            = panic "ByteCodeGen.generateCCall: missing or invalid World token?"
+            | otherwise
+            = reverse (tail a_reps_pushed_r_to_l)
+
+         -- Now: a_reps_pushed_RAW are the reps which are actually on the stack.
+         -- push_args is the code to do that.
+         -- d_after_args is the stack depth once the args are on.
+
+         -- Get the result rep.
          (returns_void, r_rep)
-            = case maybe_r_rep of
+            = case maybe_getCCallReturnRep (idType fn) of
                  Nothing -> (True,  VoidRep)
                  Just rr -> (False, rr) 
          {-
@@ -659,38 +771,38 @@ generateCCall d s fn ccall_spec@(CCallSpec target cconv safety)
             void marshall_code ( StgWord* ptr_to_top_of_stack )
          -}
          -- resolve static address
-         (is_static, static_target_addr)
+         get_target_info
             = case target of
                  DynamicTarget
-                    -> (False, panic "ByteCodeGen.generateCCall(dyn)")
+                    -> returnBc (False, panic "ByteCodeGen.generateCCall(dyn)")
                  StaticTarget target
-                    -> let unpacked = _UNPK_ target
-                       in  case unsafePerformIO (lookupSymbol unpacked) of
-                              Just aa -> case aa of Ptr a# -> (True, A# a#)
-                              Nothing -> invalid
+                    -> let sym_to_find = _UNPK_ target in
+                       ioToBc (lookupSymbol sym_to_find) `thenBc` \res ->
+                       case res of
+                           Just aa -> case aa of Ptr a# -> returnBc (True, A# a#)
+                           Nothing -> ioToBc (linkFail "ByteCodeGen.generateCCall" 
+                                                       sym_to_find)
                  CasmTarget _
-                    -> invalid
-                 where
-                    invalid = pprPanic ("ByteCodeGen.generateCCall: unfindable " 
-                                        ++ "symbol or otherwise invalid target")
-                                       (ppr ccall_spec)
+                    -> pprPanic "ByteCodeGen.generateCCall: casm" (ppr ccall_spec)
+     in
+         get_target_info       `thenBc` \ (is_static, static_target_addr) ->
+     let
 
          -- Get the arg reps, zapping the leading Addr# in the dynamic case
-         a_reps | is_static = a_reps_RAW
-                | otherwise = if null a_reps_RAW 
+         a_reps -- | trace (showSDoc (ppr a_reps_pushed_RAW)) False = error "???"
+                | is_static = a_reps_pushed_RAW
+                | otherwise = if null a_reps_pushed_RAW 
                               then panic "ByteCodeGen.generateCCall: dyn with no args"
-                              else tail a_reps_RAW
+                              else tail a_reps_pushed_RAW
 
          -- push the Addr#
-         addr_usizeW = untaggedSizeW AddrRep
-         addr_tsizeW = taggedSizeW AddrRep
          (push_Addr, d_after_Addr)
             | is_static
             = (toOL [PUSH_UBX (Right static_target_addr) addr_usizeW,
                      PUSH_TAG addr_usizeW],
-               d + addr_tsizeW)
+               d_after_args + addr_tsizeW)
             | otherwise        -- is already on the stack
-            = (nilOL, d)
+            = (nilOL, d_after_args)
 
          -- Push the return placeholder.  For a call returning nothing,
          -- this is a VoidRep (tag).
@@ -704,25 +816,29 @@ generateCCall d s fn ccall_spec@(CCallSpec target cconv safety)
                       `appOL` 
                       unitOL (PUSH_TAG r_usizeW)
 
-         -- do the call
-         do_call      = unitOL (CCALL addr_of_marshaller)
-         -- slide and return
-         wrapup       = mkSLIDE r_tsizeW (d_after_r - r_tsizeW - s)
-                        `snocOL` RETURN r_rep
-
          -- generate the marshalling code we're going to call
          r_offW       = 0 
          addr_offW    = r_tsizeW
          arg1_offW    = r_tsizeW + addr_tsizeW
          args_offW    = map (arg1_offW +) 
                             (init (scanl (+) 0 (map taggedSizeW a_reps)))
-         addr_of_marshaller
-                      = mkMarshalCode cconv
-                                      (r_offW, r_rep) addr_offW
-                                      (zip args_offW a_reps)
+     in
+         ioToBc (mkMarshalCode cconv
+                    (r_offW, r_rep) addr_offW
+                    (zip args_offW a_reps))    `thenBc` \ addr_of_marshaller ->
+         recordMallocBc addr_of_marshaller     `thenBc_`
+     let
+         -- do the call
+         do_call      = unitOL (CCALL addr_of_marshaller)
+         -- slide and return
+         wrapup       = mkSLIDE r_tsizeW (d_after_r - r_tsizeW - s)
+                        `snocOL` RETURN r_rep
      in
          --trace (show (arg1_offW, args_offW  ,  (map taggedSizeW a_reps) )) (
+         returnBc (
+         push_args `appOL`
          push_Addr `appOL` push_r `appOL` do_call `appOL` wrapup
+         )
          --)
 
 
@@ -731,55 +847,52 @@ generateCCall d s fn ccall_spec@(CCallSpec target cconv safety)
 mkDummyLiteral :: PrimRep -> Literal
 mkDummyLiteral pr
    = case pr of
+        CharRep   -> MachChar 0
         IntRep    -> MachInt 0
+        WordRep   -> MachWord 0
         DoubleRep -> MachDouble 0
         FloatRep  -> MachFloat 0
         AddrRep   | taggedSizeW AddrRep == taggedSizeW WordRep -> MachWord 0
-        _         -> pprPanic "mkDummyLiteral" (ppr pr)
+        _         -> moan64 "mkDummyLiteral" (ppr pr)
 
 
 -- Convert (eg) 
---       PrelGHC.Int# -> PrelGHC.State# PrelGHC.RealWorld
---                    -> (# PrelGHC.State# PrelGHC.RealWorld, PrelGHC.Int# #)
+--     PrelGHC.Char# -> PrelGHC.State# PrelGHC.RealWorld
+--                   -> (# PrelGHC.State# PrelGHC.RealWorld, PrelGHC.Int# #)
 --
--- to [IntRep] -> Just IntRep
--- and check that the last arg is VoidRep'd and that an unboxed pair is
--- returned wherein the first arg is VoidRep'd.
+-- to  Just IntRep
+-- and check that an unboxed pair is returned wherein the first arg is VoidRep'd.
 --
 -- Alternatively, for call-targets returning nothing, convert
 --
---       PrelGHC.Int# -> PrelGHC.State# PrelGHC.RealWorld
---                    -> (# PrelGHC.State# PrelGHC.RealWorld, PrelGHC.Int# #)
+--     PrelGHC.Char# -> PrelGHC.State# PrelGHC.RealWorld
+--                   -> (# PrelGHC.State# PrelGHC.RealWorld #)
 --
--- to [IntRep] -> Nothing
+-- to  Nothing
 
-getCCallPrimReps :: Type -> ([PrimRep], Maybe PrimRep)
-getCCallPrimReps fn_ty
+maybe_getCCallReturnRep :: Type -> Maybe PrimRep
+maybe_getCCallReturnRep fn_ty
    = let (a_tys, r_ty) = splitRepFunTys fn_ty
-         a_reps        = map typePrimRep a_tys
-         a_reps_to_go  = init a_reps
          maybe_r_rep_to_go  
-            = if length r_reps == 1 then Nothing else Just (r_reps !! 1)
+            = if isSingleton r_reps then Nothing else Just (r_reps !! 1)
          (r_tycon, r_reps) 
             = case splitTyConApp_maybe (repType r_ty) of
                       (Just (tyc, tys)) -> (tyc, map typePrimRep tys)
                       Nothing -> blargh
-
-         ok = length a_reps >= 1 && VoidRep == last a_reps
-               && ( (length r_reps == 2 && VoidRep == head r_reps)
-                    || r_reps == [VoidRep] )
-               && isUnboxedTupleTyCon r_tycon
-               && case maybe_r_rep_to_go of
-                     Nothing    -> True
-                     Just r_rep -> r_rep /= PtrRep
-                                   -- if it was, it would be impossible 
-                                   -- to create a valid return value 
-                                   -- placeholder on the stack
-         blargh       = pprPanic "getCCallPrimReps: can't handle:" 
-                                 (pprType fn_ty)
+         ok = ( ( r_reps `lengthIs` 2 && VoidRep == head r_reps)
+                || r_reps == [VoidRep] )
+              && isUnboxedTupleTyCon r_tycon
+              && case maybe_r_rep_to_go of
+                    Nothing    -> True
+                    Just r_rep -> r_rep /= PtrRep
+                                  -- if it was, it would be impossible 
+                                  -- to create a valid return value 
+                                  -- placeholder on the stack
+         blargh = pprPanic "maybe_getCCallReturn: can't handle:" 
+                           (pprType fn_ty)
      in 
      --trace (showSDoc (ppr (a_reps, r_reps))) (
-     if ok then (a_reps_to_go, maybe_r_rep_to_go) else blargh
+     if ok then maybe_r_rep_to_go else blargh
      --)
 
 atomRep (AnnVar v)    = typePrimRep (idType v)
@@ -874,10 +987,10 @@ mkUnpackCode vars d p
         code_np = do_nptrs vreps_env_uszw ptrs_szw (reverse (map snd vreps_np))
         do_nptrs off_h off_s [] = nilOL
         do_nptrs off_h off_s (npr:nprs)
-           | npr `elem` [IntRep, FloatRep, DoubleRep, CharRep, AddrRep]
+           | npr `elem` [IntRep, WordRep, FloatRep, DoubleRep, CharRep, AddrRep]
            = approved
            | otherwise
-           = pprPanic "ByteCodeGen.mkUnpackCode" (ppr npr)
+           = moan64 "ByteCodeGen.mkUnpackCode" (ppr npr)
              where
                 approved = UPK_TAG usizeW (off_h-usizeW) off_s   `consOL` theRest
                 theRest  = do_nptrs (off_h-usizeW) (off_s + tsizeW) nprs
@@ -909,18 +1022,18 @@ mkUnpackCode vars d p
 -- 5 and not to 4.  Stack locations are numbered from zero, so a depth
 -- 6 stack has valid words 0 .. 5.
 
-pushAtom :: Bool -> Int -> BCEnv -> AnnExpr' Id VarSet -> (BCInstrList, Int)
+pushAtom :: Bool -> Int -> BCEnv -> AnnExpr' Id VarSet -> BcM (BCInstrList, Int)
 pushAtom tagged d p (AnnVar v)
 
    | idPrimRep v == VoidRep
-   = ASSERT(tagged)
-     (unitOL (PUSH_TAG 0), 1)
+   = if tagged then returnBc (unitOL (PUSH_TAG 0), 1) 
+               else panic "ByteCodeGen.pushAtom(VoidRep,untaggedly)"
 
    | isFCallId v
    = pprPanic "pushAtom: shouldn't get an FCallId here" (ppr v)
 
    | Just primop <- isPrimOpId_maybe v
-   = (unitOL (PUSH_G (Right primop)), 1)
+   = returnBc (unitOL (PUSH_G (Right primop)), 1)
 
    | otherwise
    = let  {-
@@ -947,11 +1060,11 @@ pushAtom tagged d p (AnnVar v)
          sz_u   = untaggedIdSizeW v
          nwords = if tagged then sz_t else sz_u
      in
-         result
+         returnBc result
 
 pushAtom True d p (AnnLit lit)
-   = let (ubx_code, ubx_size) = pushAtom False d p (AnnLit lit)
-     in  (ubx_code `snocOL` PUSH_TAG ubx_size, 1 + ubx_size)
+   = pushAtom False d p (AnnLit lit)           `thenBc` \ (ubx_code, ubx_size) ->
+     returnBc (ubx_code `snocOL` PUSH_TAG ubx_size, 1 + ubx_size)
 
 pushAtom False d p (AnnLit lit)
    = case lit of
@@ -964,12 +1077,13 @@ pushAtom False d p (AnnLit lit)
      where
         code rep
            = let size_host_words = untaggedSizeW rep
-             in (unitOL (PUSH_UBX (Left lit) size_host_words), size_host_words)
+             in  returnBc (unitOL (PUSH_UBX (Left lit) size_host_words), 
+                           size_host_words)
 
         pushStr s 
-           = let mallocvilleAddr
+           = let getMallocvilleAddr
                     = case s of
-                         CharStr s i -> A# s
+                         CharStr s i -> returnBc (A# s)
 
                          FastString _ l ba -> 
                             -- sigh, a string in the heap is no good to us.
@@ -979,16 +1093,18 @@ pushAtom False d p (AnnLit lit)
                             -- at the same time.
                             let n = I# l
                             -- CAREFUL!  Chars are 32 bits in ghc 4.09+
-                            in  unsafePerformIO (
-                                   do (Ptr a#) <- mallocBytes (n+1)
-                                      strncpy (Ptr a#) ba (fromIntegral n)
+                            in  ioToBc (mallocBytes (n+1)) `thenBc` \ (Ptr a#) ->
+                                recordMallocBc (A# a#)     `thenBc_`
+                                ioToBc (
+                                   do strncpy (Ptr a#) ba (fromIntegral n)
                                       writeCharOffAddr (A# a#) n '\0'
                                       return (A# a#)
                                    )
-                         _ -> panic "StgInterp.lit2expr: unhandled string constant type"
+                         other -> panic "ByteCodeGen.pushAtom.pushStr"
              in
+                getMallocvilleAddr `thenBc` \ addr ->
                 -- Get the addr on the stack, untaggedly
-                (unitOL (PUSH_UBX (Right mallocvilleAddr) 1), 1)
+                   returnBc (unitOL (PUSH_UBX (Right addr) 1), 1)
 
 
 
@@ -1183,23 +1299,34 @@ bind x f    = f x
 \begin{code}
 data BcM_State 
    = BcM_State { bcos      :: [ProtoBCO Name], -- accumulates completed BCOs
-                 nextlabel :: Int }            -- for generating local labels
+                 nextlabel :: Int,             -- for generating local labels
+                 malloced  :: [Addr] }         -- ptrs malloced for current BCO
+                                                -- Should be free()d when it is GCd
+type BcM r = BcM_State -> IO (BcM_State, r)
 
-type BcM result = BcM_State -> (result, BcM_State)
+ioToBc :: IO a -> BcM a
+ioToBc io st = do x <- io 
+                  return (st, x)
 
-runBc :: BcM_State -> BcM () -> BcM_State
-runBc init_st m = case m init_st of { (r,st) -> st }
+runBc :: BcM_State -> BcM r -> IO (BcM_State, r)
+runBc st0 m = do (st1, res) <- m st0
+                 return (st1, res)
 
 thenBc :: BcM a -> (a -> BcM b) -> BcM b
-thenBc expr cont st
-  = case expr st of { (result, st') -> cont result st' }
+thenBc expr cont st0
+   = do (st1, q) <- expr st0
+        (st2, r) <- cont q st1
+        return (st2, r)
 
 thenBc_ :: BcM a -> BcM b -> BcM b
-thenBc_ expr cont st
-  = case expr st of { (result, st') -> cont st' }
+thenBc_ expr cont st0
+   = do (st1, q) <- expr st0
+        (st2, r) <- cont st1
+        return (st2, r)
 
 returnBc :: a -> BcM a
-returnBc result st = (result, st)
+returnBc result st = return (st, result)
+
 
 mapBc :: (a -> BcM b) -> [a] -> BcM [b]
 mapBc f []     = returnBc []
@@ -1208,17 +1335,28 @@ mapBc f (x:xs)
     mapBc f xs   `thenBc` \ rs ->
     returnBc (r:rs)
 
-emitBc :: ProtoBCO Name -> BcM ()
+emitBc :: ([Addr] -> ProtoBCO Name) -> BcM ()
 emitBc bco st
-   = ((), st{bcos = bco : bcos st})
+   = return (st{bcos = bco (malloced st) : bcos st, malloced=[]}, ())
+
+newbcoBc :: BcM ()
+newbcoBc st
+   | not (null (malloced st)) 
+   = panic "ByteCodeGen.newbcoBc: missed prior emitBc?"
+   | otherwise
+   = return (st, ())
+
+recordMallocBc :: Addr -> BcM ()
+recordMallocBc a st
+   = return (st{malloced = a : malloced st}, ())
 
 getLabelBc :: BcM Int
 getLabelBc st
-   = (nextlabel st, st{nextlabel = 1 + nextlabel st})
+   = return (st{nextlabel = 1 + nextlabel st}, nextlabel st)
 
 getLabelsBc :: Int -> BcM [Int]
 getLabelsBc n st
    = let ctr = nextlabel st 
-     in  ([ctr .. ctr+n-1], st{nextlabel = ctr+n})
+     in return (st{nextlabel = ctr+n}, [ctr .. ctr+n-1])
 
 \end{code}