[project @ 2001-02-15 14:30:35 by sewardj]
[ghc-hetmet.git] / ghc / compiler / ghci / ByteCodeGen.lhs
index 0a77cbf..cea9dbb 100644 (file)
@@ -4,62 +4,70 @@
 \section[ByteCodeGen]{Generate bytecode from Core}
 
 \begin{code}
-module ByteCodeGen ( byteCodeGen, linkIModules ) where
+module ByteCodeGen ( UnlinkedBCO, UnlinkedBCOExpr, ItblEnv, ClosureEnv, HValue,
+                    filterNameMap,
+                     byteCodeGen, coreExprToBCOs, 
+                    linkIModules, linkIExpr
+                  ) where
 
 #include "HsVersions.h"
 
 import Outputable
-import Name            ( Name, getName )
-import Id              ( Id, idType, isDataConId_maybe )
+import Name            ( Name, getName, mkSysLocalName )
+import Id              ( Id, idType, isDataConId_maybe, mkVanillaId,
+                         isPrimOpId_maybe, idPrimRep )
 import OrdList         ( OrdList, consOL, snocOL, appOL, unitOL, 
                          nilOL, toOL, concatOL, fromOL )
-import FiniteMap       ( FiniteMap, addListToFM, listToFM, 
-                         addToFM, lookupFM, fmToList, emptyFM, plusFM )
+import FiniteMap       ( FiniteMap, addListToFM, listToFM,
+                         addToFM, lookupFM, fmToList, plusFM )
 import CoreSyn
-import PprCore         ( pprCoreExpr, pprCoreAlt )
-import Literal         ( Literal(..) )
+import PprCore         ( pprCoreExpr )
+import Literal         ( Literal(..), literalPrimRep )
 import PrimRep         ( PrimRep(..) )
+import PrimOp          ( PrimOp(..)  )
 import CoreFVs         ( freeVars )
 import Type            ( typePrimRep )
-import DataCon         ( DataCon, dataConTag, fIRST_TAG, dataConTyCon, 
-                         dataConRepArgTys )
-import TyCon           ( TyCon, tyConFamilySize, isDataTyCon, tyConDataCons )
+import DataCon         ( dataConTag, fIRST_TAG, dataConTyCon, 
+                          dataConWrapId, isUnboxedTupleCon )
+import TyCon           ( TyCon, tyConFamilySize )
 import Class           ( Class, classTyCon )
-import Util            ( zipEqual, zipWith4Equal, naturalMergeSortLe, nOfThem, global )
+import Util            ( zipEqual, zipWith4Equal, naturalMergeSortLe, nOfThem )
 import Var             ( isTyVar )
 import VarSet          ( VarSet, varSetElems )
 import PrimRep         ( getPrimRepSize, isFollowableRep )
-import Constants       ( wORD_SIZE )
 import CmdLineOpts     ( DynFlags, DynFlag(..) )
 import ErrUtils                ( showPass, dumpIfSet_dyn )
-import ClosureInfo     ( mkVirtHeapOffsets )
-
-import List            ( intersperse )
-import Monad           ( foldM )
-import ST              ( runST )
-import MArray          ( MArray(..), IOArray, IOUArray, HasBounds(..), freeze, 
-                         mapArray,
-                         castSTUArray, readWord32Array,
-                         newFloatArray, writeFloatArray,
-                         newDoubleArray,  writeDoubleArray,
-                         newIntArray, writeIntArray,
-                         newAddrArray, writeAddrArray )
-import Foreign         ( Storable(..), Word8, Word16, Word32, Ptr(..), 
-                         malloc, castPtr, plusPtr )
-import Addr            ( Addr, addrToInt, nullAddr )
-import Bits            ( Bits(..), shiftR )
-
-import PrelGHC         ( BCO#, newBCO#, unsafeCoerce#, ByteArray#, Array# )
-import IOExts          ( IORef, readIORef, writeIORef, fixIO )
-import ArrayBase       
-import PrelArr         ( Array(..) )
+import Unique          ( mkPseudoUnique3 )
+import FastString      ( FastString(..) )
+import Panic           ( GhcException(..) )
+import PprType         ( pprType )
+import ByteCodeInstr   ( BCInstr(..), ProtoBCO(..), nameOfProtoBCO, bciStackUse )
+import ByteCodeItbls   ( ItblEnv, mkITbls )
+import ByteCodeLink    ( UnlinkedBCO, UnlinkedBCOExpr, assembleBCO,
+                         ClosureEnv, HValue, linkSomeBCOs, filterNameMap,
+                         iNTERP_STACK_CHECK_THRESH )
+
+import List            ( intersperse, sortBy )
+import Foreign         ( Ptr(..), mallocBytes )
+import Addr            ( Addr(..), addrToInt, writeCharOffAddr )
+import CTypes          ( CInt )
+import Exception       ( throwDyn )
+
+import PrelBase                ( Int(..) )
+import PrelGHC         ( ByteArray# )
+import IOExts          ( unsafePerformIO )
 import PrelIOBase      ( IO(..) )
+
 \end{code}
 
-Entry point.
+%************************************************************************
+%*                                                                     *
+\subsection{Functions visible from outside this module.}
+%*                                                                     *
+%************************************************************************
 
 \begin{code}
--- visible from outside
+
 byteCodeGen :: DynFlags
             -> [CoreBind] 
             -> [TyCon] -> [Class]
@@ -73,7 +81,8 @@ byteCodeGen dflags binds local_tycons local_classes
             getBind (NonRec bndr rhs) = [(bndr, freeVars rhs)]
             getBind (Rec binds)       = [(bndr, freeVars rhs) | (bndr,rhs) <- binds]
             final_state = runBc (BcM_State [] 0) 
-                                (mapBc schemeR flatBinds `thenBc_` returnBc ())
+                                (mapBc (schemeR True) flatBinds
+                                       `thenBc_` returnBc ())
             (BcM_State proto_bcos final_ctr) = final_state
 
         dumpIfSet_dyn dflags Opt_D_dump_BCOs
@@ -84,117 +93,56 @@ byteCodeGen dflags binds local_tycons local_classes
         return (bcos, itblenv)
         
 
-data UnlinkedBCO
-   = UnlinkedBCO Name
-                 Int (IOUArray Int Word16)     -- insns
-                 Int (IOUArray Int Word32)     -- literals
-                 Int (IOArray Int Name)                -- ptrs
-                 Int (IOArray Int Name)                -- itbl refs
+-- Returns: (the root BCO for this expression, 
+--           a list of auxilary BCOs resulting from compiling closures)
+coreExprToBCOs :: DynFlags
+              -> CoreExpr
+               -> IO UnlinkedBCOExpr
+coreExprToBCOs dflags expr
+ = do showPass dflags "ByteCodeGen"
 
-nameOfUnlinkedBCO (UnlinkedBCO nm _ _ _ _ _ _ _ _) = nm
+      -- create a totally bogus name for the top-level BCO; this
+      -- should be harmless, since it's never used for anything
+      let invented_name = mkSysLocalName (mkPseudoUnique3 0) SLIT("Expr-Top-Level")
+      let invented_id   = mkVanillaId invented_name (panic "invented_id's type")
 
--- needs a proper home
-type ItblEnv    = FiniteMap Name (Ptr StgInfoTable)
-type ClosureEnv = FiniteMap Name HValue
-data HValue = HValue  -- dummy type, actually a pointer to some Real Code.
+      let (BcM_State all_proto_bcos final_ctr) 
+             = runBc (BcM_State [] 0) 
+                     (schemeR True (invented_id, freeVars expr))
+      dumpIfSet_dyn dflags Opt_D_dump_BCOs
+         "Proto-bcos" (vcat (intersperse (char ' ') (map ppr all_proto_bcos)))
 
-\end{code}
+      let root_proto_bco 
+             = case filter ((== invented_name).nameOfProtoBCO) all_proto_bcos of
+                  [root_bco] -> root_bco
+          auxiliary_proto_bcos
+             = filter ((/= invented_name).nameOfProtoBCO) all_proto_bcos
 
+      auxiliary_bcos <- mapM assembleBCO auxiliary_proto_bcos
+      root_bco <- assembleBCO root_proto_bco
 
-%************************************************************************
-%*                                                                     *
-\subsection{Bytecodes, and Outputery.}
-%*                                                                     *
-%************************************************************************
+      return (root_bco, auxiliary_bcos)
 
-\begin{code}
 
-type LocalLabel = Int
-
-data UnboxedLit = UnboxedI Int | UnboxedF Float | UnboxedD Double
-
-data BCInstr
-   -- Messing with the stack
-   = ARGCHECK  Int
-   -- Push locals (existing bits of the stack)
-   | PUSH_L    Int{-offset-}
-   | PUSH_LL   Int Int{-2 offsets-}
-   | PUSH_LLL  Int Int Int{-3 offsets-}
-   -- Push a ptr
-   | PUSH_G    Name
-   -- Push an alt continuation
-   | PUSH_AS   Name PrimRep    -- push alts and BCO_ptr_ret_info
-                               -- PrimRep so we know which itbl
-   -- Pushing literals
-   | PUSH_UBX  Literal Int 
-                        -- push this int/float/double, NO TAG, on the stack
-                       -- Int is # of items in literal pool to push
-   | PUSH_TAG  Int      -- push this tag on the stack
-
-   | SLIDE     Int{-this many-} Int{-down by this much-}
-   -- To do with the heap
-   | ALLOC     Int     -- make an AP_UPD with this many payload words, zeroed
-   | MKAP      Int{-ptr to AP_UPD is this far down stack-} Int{-# words-}
-   | UNPACK    Int     -- unpack N ptr words from t.o.s Constr
-   | UPK_TAG   Int Int Int
-                       -- unpack N non-ptr words from offset M in constructor
-                       -- K words down the stack
-   | PACK      DataCon Int
-                       -- after assembly, the DataCon is an index into the
-                       -- itbl array
-   -- For doing case trees
-   | LABEL     LocalLabel
-   | TESTLT_I  Int    LocalLabel
-   | TESTEQ_I  Int    LocalLabel
-   | TESTLT_F  Float  LocalLabel
-   | TESTEQ_F  Float  LocalLabel
-   | TESTLT_D  Double LocalLabel
-   | TESTEQ_D  Double LocalLabel
-   | TESTLT_P  Int    LocalLabel
-   | TESTEQ_P  Int    LocalLabel
-   | CASEFAIL
-   -- To Infinity And Beyond
-   | ENTER
-   | RETURN    -- unboxed value on TOS.  Use tag to find underlying ret itbl
-               -- and return as per that.
-
-
-instance Outputable BCInstr where
-   ppr (ARGCHECK n)          = text "ARGCHECK" <+> int n
-   ppr (PUSH_L offset)       = text "PUSH_L  " <+> int offset
-   ppr (PUSH_LL o1 o2)       = text "PUSH_LL " <+> int o1 <+> int o2
-   ppr (PUSH_LLL o1 o2 o3)   = text "PUSH_LLL" <+> int o1 <+> int o2 <+> int o3
-   ppr (PUSH_G nm)           = text "PUSH_G  " <+> ppr nm
-   ppr (PUSH_AS nm pk)       = text "PUSH_AS " <+> ppr nm <+> ppr pk
-   ppr (SLIDE n d)           = text "SLIDE   " <+> int n <+> int d
-   ppr (ALLOC sz)            = text "ALLOC   " <+> int sz
-   ppr (MKAP offset sz)      = text "MKAP    " <+> int offset <+> int sz
-   ppr (UNPACK sz)           = text "UNPACK  " <+> int sz
-   ppr (PACK dcon sz)        = text "PACK    " <+> ppr dcon <+> ppr sz
-   ppr (LABEL     lab)       = text "__"       <> int lab <> colon
-   ppr (TESTLT_I  i lab)     = text "TESTLT_I" <+> int i <+> text "__" <> int lab
-   ppr (TESTEQ_I  i lab)     = text "TESTEQ_I" <+> int i <+> text "__" <> int lab
-   ppr (TESTLT_F  f lab)     = text "TESTLT_F" <+> float f <+> text "__" <> int lab
-   ppr (TESTEQ_F  f lab)     = text "TESTEQ_F" <+> float f <+> text "__" <> int lab
-   ppr (TESTLT_D  d lab)     = text "TESTLT_D" <+> double d <+> text "__" <> int lab
-   ppr (TESTEQ_D  d lab)     = text "TESTEQ_D" <+> double d <+> text "__" <> int lab
-   ppr (TESTLT_P  i lab)     = text "TESTLT_P" <+> int i <+> text "__" <> int lab
-   ppr (TESTEQ_P  i lab)     = text "TESTEQ_P" <+> int i <+> text "__" <> int lab
-   ppr CASEFAIL              = text "CASEFAIL"
-   ppr ENTER                 = text "ENTER"
-   ppr RETURN                = text "RETURN"
-
-pprAltCode discrs_n_codes
-   = vcat (map f discrs_n_codes)
-     where f (discr, code) = ppr discr <> colon <+> vcat (map ppr (fromOL code))
-
-instance Outputable a => Outputable (ProtoBCO a) where
-   ppr (ProtoBCO name instrs origin)
-      = (text "ProtoBCO" <+> ppr name <> colon)
-        $$ nest 6 (vcat (map ppr instrs))
-        $$ case origin of
-              Left alts -> vcat (map (pprCoreAlt.deAnnAlt) alts)
-              Right rhs -> pprCoreExpr (deAnnotate rhs)
+-- Linking stuff
+linkIModules :: ItblEnv    -- incoming global itbl env; returned updated
+            -> ClosureEnv -- incoming global closure env; returned updated
+            -> [([UnlinkedBCO], ItblEnv)]
+            -> IO ([HValue], ItblEnv, ClosureEnv)
+linkIModules gie gce mods 
+   = do let (bcoss, ies) = unzip mods
+            bcos = concat bcoss
+            final_gie = foldr plusFM gie ies
+        (final_gce, linked_bcos) <- linkSomeBCOs True final_gie gce bcos
+        return (linked_bcos, final_gie, final_gce)
+
+
+linkIExpr :: ItblEnv -> ClosureEnv -> UnlinkedBCOExpr
+          -> IO HValue           -- IO BCO# really
+linkIExpr ie ce (root_ul_bco, aux_ul_bcos)
+   = do (aux_ce, _) <- linkSomeBCOs False ie ce aux_ul_bcos
+        (_, [root_bco]) <- linkSomeBCOs False ie aux_ce [root_ul_bco]
+        return root_bco
 \end{code}
 
 %************************************************************************
@@ -207,30 +155,53 @@ instance Outputable a => Outputable (ProtoBCO a) where
 
 type BCInstrList = OrdList BCInstr
 
-data ProtoBCO a 
-   = ProtoBCO a                        -- name, in some sense
-              [BCInstr]                -- instrs
-                                       -- what the BCO came from
-              (Either [AnnAlt Id VarSet]
-                      (AnnExpr Id VarSet))
-
-
 type Sequel = Int      -- back off to this depth before ENTER
 
 -- Maps Ids to the offset from the stack _base_ so we don't have
 -- to mess with it after each push/pop.
 type BCEnv = FiniteMap Id Int  -- To find vars on the stack
 
+ppBCEnv :: BCEnv -> SDoc
+ppBCEnv p
+   = text "begin-env"
+     $$ nest 4 (vcat (map pp_one (sortBy cmp_snd (fmToList p))))
+     $$ text "end-env"
+     where
+        pp_one (var, offset) = int offset <> colon <+> ppr var
+        cmp_snd x y = compare (snd x) (snd y)
 
 -- Create a BCO and do a spot of peephole optimisation on the insns
 -- at the same time.
 mkProtoBCO nm instrs_ordlist origin
-   = ProtoBCO nm (peep (fromOL instrs_ordlist)) origin
+   = ProtoBCO nm maybe_with_stack_check origin
      where
+        -- Overestimate the stack usage (in words) of this BCO,
+        -- and if >= iNTERP_STACK_CHECK_THRESH, add an explicit
+        -- stack check.  (The interpreter always does a stack check
+        -- for iNTERP_STACK_CHECK_THRESH words at the start of each
+        -- BCO anyway, so we only need to add an explicit on in the
+        -- (hopefully rare) cases when the (overestimated) stack use
+        -- exceeds iNTERP_STACK_CHECK_THRESH.
+        maybe_with_stack_check
+           | stack_overest >= 65535
+           = pprPanic "mkProtoBCO: stack use won't fit in 16 bits" 
+                      (int stack_overest)
+           | stack_overest >= iNTERP_STACK_CHECK_THRESH
+           = (STKCHECK stack_overest) : peep_d
+           | otherwise
+           = peep_d    -- the supposedly common case
+             
+        stack_overest = sum (map bciStackUse peep_d)
+                        + 10 {- just to be really really sure -}
+
+
+        -- Merge local pushes
+        peep_d = peep (fromOL instrs_ordlist)
+
         peep (PUSH_L off1 : PUSH_L off2 : PUSH_L off3 : rest)
            = PUSH_LLL off1 (off2-1) (off3-2) : peep rest
         peep (PUSH_L off1 : PUSH_L off2 : rest)
-           = PUSH_LL off1 off2 : peep rest
+           = PUSH_LL off1 (off2-1) : peep rest
         peep (i:rest)
            = i : peep rest
         peep []
@@ -240,25 +211,63 @@ mkProtoBCO nm instrs_ordlist origin
 -- Compile code for the right hand side of a let binding.
 -- Park the resulting BCO in the monad.  Also requires the
 -- variable to which this value was bound, so as to give the
--- resulting BCO a name.
-schemeR :: (Id, AnnExpr Id VarSet) -> BcM ()
-schemeR (nm, rhs) = schemeR_wrk rhs nm (collect [] rhs)
+-- resulting BCO a name.  Bool indicates top-levelness.
+
+schemeR :: Bool -> (Id, AnnExpr Id VarSet) -> BcM ()
+schemeR is_top (nm, rhs) 
+{-
+   | trace (showSDoc (
+              (char ' '
+               $$ (ppr.filter (not.isTyVar).varSetElems.fst) rhs
+               $$ pprCoreExpr (deAnnotate rhs)
+               $$ char ' '
+              ))) False
+   = undefined
+-}
+   | otherwise
+   = schemeR_wrk is_top rhs nm (collect [] rhs)
 
+
+collect xs (_, AnnNote note e)
+   = collect xs e
 collect xs (_, AnnLam x e) 
    = collect (if isTyVar x then xs else (x:xs)) e
 collect xs not_lambda
    = (reverse xs, not_lambda)
 
-schemeR_wrk original_body nm (args, body)
+schemeR_wrk is_top 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])
+                                     (Right original_body))
+     --)
+
+   | otherwise
    = let fvs       = filter (not.isTyVar) (varSetElems (fst original_body))
-         all_args  = fvs ++ reverse args
+         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))
-         argcheck  = if null args then nilOL else unitOL (ARGCHECK szw_args)
+         argcheck  = unitOL (ARGCHECK szw_args)
      in
      schemeE szw_args 0 p_init body            `thenBc` \ body_code ->
-     emitBc (mkProtoBCO (getName nm) (appOL argcheck body_code) (Right original_body))
+     emitBc (mkProtoBCO (getName nm) (appOL argcheck body_code) 
+                                     (Right original_body))
+
+     where
+        maybe_toplevel_null_con_rhs
+           | is_top && null args
+           = case snd body of
+                AnnVar v_wrk 
+                   -> case isDataConId_maybe v_wrk of
+                         Nothing -> Nothing
+                         Just dc_wrk |  nm == dataConWrapId dc_wrk
+                                     -> Just dc_wrk
+                                     |  otherwise 
+                                     -> Nothing
+                other -> Nothing
+           | otherwise
+           = Nothing
 
 -- 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
@@ -273,28 +282,34 @@ schemeE :: Int -> Sequel -> BCEnv -> AnnExpr Id VarSet -> BcM BCInstrList
 
 -- Delegate tail-calls to schemeT.
 schemeE d s p e@(fvs, AnnApp f a) 
-   = returnBc (schemeT (should_args_be_tagged e) d s 0 p (fvs, AnnApp f a))
+   = returnBc (schemeT d s p (fvs, AnnApp f a))
 schemeE d s p e@(fvs, AnnVar v)
-   | isFollowableRep (typePrimRep (idType v))
-   = returnBc (schemeT (should_args_be_tagged e) d s 0 p (fvs, AnnVar v))
+   | isFollowableRep v_rep
+   = returnBc (schemeT d s p (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
-                   `snocOL` SLIDE szw (d-s)    -- clear to sequel
-                   `snocOL` RETURN)            -- go
+                   `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
      in  returnBc (push                        -- value onto stack
-                   `snocOL` SLIDE szw (d-s)    -- clear to sequel
-                   `snocOL` RETURN)            -- go
+                   `appOL`  mkSLIDE szw (d-s)  -- clear to sequel
+                   `snocOL` RETURN l_rep)      -- go
 
 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
+
+         -- Sizes of tagged free vars, + 1 for the fn
          sizes = map (\rhs_fvs -> 1 + sum (map taggedIdSizeW rhs_fvs)) fvss
 
          -- This p', d' defn is safe because all the items being pushed
@@ -310,7 +325,7 @@ 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 (getName id) 
+            = 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
@@ -322,7 +337,7 @@ schemeE d s p (fvs, AnnLet binds b)
          allocCode = toOL (map ALLOC sizes)
      in
      schemeE d' s p' b                                 `thenBc`  \ bodyCode ->
-     mapBc schemeR (zip xs rhss)                       `thenBc_`
+     mapBc (schemeR False) (zip xs rhss)               `thenBc_`
      returnBc (allocCode `appOL` thunkCode `appOL` bodyCode)
 
 
@@ -342,33 +357,37 @@ schemeE d s p (fvs, AnnCase scrut bndr alts)
         scrut_primrep = typePrimRep (idType bndr)
         isAlgCase
            = case scrut_primrep of
+                CharRep -> False ; AddrRep -> False ; WordRep -> False
                 IntRep -> False ; FloatRep -> False ; DoubleRep -> False
+                VoidRep -> False ;
                 PtrRep -> True
                 other  -> pprPanic "ByteCodeGen.schemeE" (ppr other)
 
         -- given an alt, return a discr and code for it.
         codeAlt alt@(discr, binds_f, rhs)
            | isAlgCase 
-           = let binds_r      = reverse binds_f
-                 binds_r_szsw = map untaggedIdSizeW binds_r
-                 binds_szw    = sum binds_r_szsw
-                 p''          = addListToFM 
-                                   p' (zip binds_r (mkStackOffsets d' binds_r_szsw))
-                 d''          = d' + binds_szw
-                 unpack_code  = mkUnpackCode 0 0 (map (typePrimRep.idType) binds_f)
-             in schemeE d'' s p'' rhs  `thenBc` \ rhs_code -> 
-                returnBc (my_discr alt, unpack_code `appOL` rhs_code)
+           = let (unpack_code, d_after_unpack, p_after_unpack)
+                    = mkUnpackCode binds_f d' p'
+             in  schemeE d_after_unpack s p_after_unpack rhs
+                                       `thenBc` \ rhs_code -> 
+                 returnBc (my_discr alt, unpack_code `appOL` rhs_code)
            | otherwise 
            = ASSERT(null binds_f) 
              schemeE d' s p' rhs       `thenBc` \ rhs_code ->
              returnBc (my_discr alt, rhs_code)
 
-        my_discr (DEFAULT, binds, rhs)  = NoDiscr
-        my_discr (DataAlt dc, binds, rhs) = DiscrP (dataConTag dc)
+        my_discr (DEFAULT, binds, rhs) = NoDiscr
+        my_discr (DataAlt dc, binds, rhs) 
+           | isUnboxedTupleCon dc
+           = unboxedTupleException
+           | otherwise
+           = DiscrP (dataConTag dc - fIRST_TAG)
         my_discr (LitAlt l, binds, rhs)
            = case l of MachInt i     -> DiscrI (fromInteger i)
                        MachFloat r   -> DiscrF (fromRational r)
                        MachDouble r  -> DiscrD (fromRational r)
+                       MachChar i    -> DiscrI i
+                       _ -> pprPanic "schemeE(AnnCase).my_discr" (ppr l)
 
         maybe_ncons 
            | not isAlgCase = Nothing
@@ -381,8 +400,9 @@ schemeE d s p (fvs, AnnCase scrut bndr alts)
      mapBc codeAlt alts                                `thenBc` \ alt_stuff ->
      mkMultiBranch maybe_ncons alt_stuff               `thenBc` \ alt_final ->
      let 
+         alt_final_ac = ARGCHECK (taggedIdSizeW bndr) `consOL` alt_final
          alt_bco_name = getName bndr
-         alt_bco      = mkProtoBCO alt_bco_name alt_final (Left alts)
+         alt_bco      = mkProtoBCO alt_bco_name alt_final_ac (Left alts)
      in
      schemeE (d + ret_frame_sizeW) 
              (d + ret_frame_sizeW) p scrut             `thenBc` \ scrut_code ->
@@ -399,71 +419,171 @@ schemeE d s p other
                (pprCoreExpr (deAnnotate other))
 
 
--- Compile code to do a tail call.  Doesn't need to be monadic.
-schemeT :: Bool        -- do tagging?
-        -> Int                 -- Stack depth
+-- Compile code to do a tail call.  Three cases:
+--
+-- 1.  A nullary constructor.  Push its closure on the stack 
+--     and SLIDE and RETURN.
+--
+-- 2.  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.
+--
+-- 3.  Otherwise, it must be a function call.  Push the args
+--     right to left, SLIDE and ENTER.
+
+schemeT :: Int                 -- Stack depth
         -> Sequel      -- Sequel depth
-        -> Int                 -- # arg words so far
         -> BCEnv       -- stack env
         -> AnnExpr Id VarSet 
         -> BCInstrList
 
-schemeT enTag d s narg_words p (_, AnnApp f a)
-   = case snd a of
-        AnnType _ -> schemeT enTag d s narg_words p f
-        other
-           -> let (push, arg_words) = pushAtom enTag d p (snd a)
-              in push 
-                 `appOL` schemeT enTag (d+arg_words) s (narg_words+arg_words) p f
-
-schemeT enTag d s narg_words p (_, AnnVar f)
-   | Just con <- isDataConId_maybe f
-   = ASSERT(enTag == False)
-     PACK con narg_words `consOL` (mkSLIDE 1 (d-s-1) `snocOL` ENTER)
+schemeT d s p app
+--   | trace ("schemeT: env in = \n" ++ showSDocDebug (ppBCEnv p)) False
+--   = panic "schemeT ?!?!"
+
+   -- Handle case 1
+   | is_con_call && null args_r_to_l
+   = (PUSH_G (Left (getName con)) `consOL` mkSLIDE 1 (d-s))
+     `snocOL` ENTER
+
+   -- Cases 2 and 3
    | otherwise
-   = ASSERT(enTag == True)
-     let (push, arg_words) = pushAtom True d p (AnnVar f)
-     in  push 
-         `appOL`  mkSLIDE (narg_words+arg_words) (d - s - narg_words)
-         `snocOL` ENTER
+   = if   is_con_call && isUnboxedTupleCon con
+     then unboxedTupleException
+     else code
+
+     where
+         -- Extract the args (R->L) and fn
+         (args_r_to_l_raw, fn) = chomp app
+         chomp expr
+            = case snd expr of
+                 AnnVar v    -> ([], v)
+                 AnnApp f a  -> case chomp f of (az, f) -> (snd a:az, f)
+                 AnnNote n e -> chomp e
+                 other       -> pprPanic "schemeT" 
+                                   (ppr (deAnnotate (panic "schemeT.chomp", other)))
+         
+         args_r_to_l = filter (not.isTypeAtom) args_r_to_l_raw
+         isTypeAtom (AnnType _) = True
+         isTypeAtom _           = False
+
+         -- decide if this is a constructor call, and rearrange
+         -- args appropriately.
+         maybe_dcon  = isDataConId_maybe fn
+         is_con_call = case maybe_dcon of Nothing -> False; Just _ -> True
+         (Just con)  = maybe_dcon
+
+         args_final_r_to_l
+            | not is_con_call
+            = args_r_to_l
+            | otherwise
+            = filter (not.isPtr) args_r_to_l ++ filter isPtr args_r_to_l
+              where isPtr = isFollowableRep . atomRep
+
+         -- make code to push the args and then do the SLIDE-ENTER thing
+         code = do_pushery d args_final_r_to_l
+
+         tag_when_push = not is_con_call
+         narg_words    = sum (map (get_arg_szw . atomRep) 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
+         do_pushery d []
+            = case maybe_dcon of
+                 Just con -> 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
 
 mkSLIDE n d 
    = if d == 0 then nilOL else unitOL (SLIDE n d)
 
-should_args_be_tagged (_, AnnVar v)
-   = case isDataConId_maybe v of
-        Just dcon -> False; Nothing -> True
-should_args_be_tagged (_, AnnApp f a)
-   = should_args_be_tagged f
-should_args_be_tagged (_, other)
-   = panic "should_args_be_tagged: tail call to non-con, non-var"
-
-
--- Make code to unpack a constructor onto the stack, adding
--- tags for the unboxed bits.  Takes the PrimReps of the constructor's
--- arguments, and a travelling offset along both the constructor
--- (off_h) and the stack (off_s).
-mkUnpackCode :: Int -> Int -> [PrimRep] -> BCInstrList
-mkUnpackCode off_h off_s [] = nilOL
-mkUnpackCode off_h off_s (r:rs)
-   | isFollowableRep r
-   = let (rs_ptr, rs_nptr) = span isFollowableRep (r:rs)
-         ptrs_szw = sum (map untaggedSizeW rs_ptr) 
-     in  ASSERT(ptrs_szw == length rs_ptr)
-         ASSERT(off_h == 0)
-         ASSERT(off_s == 0)
-         UNPACK ptrs_szw 
-         `consOL` mkUnpackCode (off_h + ptrs_szw) (off_s + ptrs_szw) rs_nptr
-   | otherwise
-   = case r of
-        IntRep    -> approved
-        FloatRep  -> approved
-        DoubleRep -> approved
+atomRep (AnnVar v)    = typePrimRep (idType v)
+atomRep (AnnLit l)    = literalPrimRep l
+atomRep (AnnNote n b) = atomRep (snd b)
+atomRep (AnnApp f (_, AnnType _)) = atomRep (snd f)
+atomRep (AnnLam x e) | isTyVar x = atomRep (snd e)
+atomRep other = pprPanic "atomRep" (ppr (deAnnotate (undefined,other)))
+
+
+-- Make code to unpack the top-of-stack constructor onto the stack, 
+-- adding tags for the unboxed bits.  Takes the PrimReps of the 
+-- constructor's arguments.  off_h and off_s are travelling offsets
+-- along the constructor and the stack.
+--
+-- Supposing a constructor in the heap has layout
+--
+--      Itbl p_1 ... p_i np_1 ... np_j
+--
+-- then we add to the stack, shown growing down, the following:
+--
+--    (previous stack)
+--         p_i
+--         ...
+--         p_1
+--         np_j
+--         tag_for(np_j)
+--         ..
+--         np_1
+--         tag_for(np_1)
+--
+-- so that in the common case (ptrs only) a single UNPACK instr can
+-- copy all the payload of the constr onto the stack with no further ado.
+
+mkUnpackCode :: [Id]   -- constr args
+             -> Int    -- depth before unpack
+             -> BCEnv  -- env before unpack
+             -> (BCInstrList, Int, BCEnv)
+mkUnpackCode vars d p
+   = --trace ("mkUnpackCode: " ++ showSDocDebug (ppr vars)
+     --       ++ " --> " ++ show d' ++ "\n" ++ showSDocDebug (ppBCEnv p')
+     --       ++ "\n") (
+     (code_p `appOL` code_np, d', p')
+     --)
      where
-        approved = UPK_TAG usizeW off_h off_s   `consOL` theRest
-        theRest  = mkUnpackCode (off_h + usizeW) (off_s + tsizeW) rs
-        usizeW   = untaggedSizeW r
-        tsizeW   = taggedSizeW r
+        -- vars with reps
+        vreps = [(var, typePrimRep (idType var)) | var <- vars]
+
+        -- ptrs and nonptrs, forward
+        vreps_p  = filter (isFollowableRep.snd) vreps
+        vreps_np = filter (not.isFollowableRep.snd) vreps
+
+        -- the order in which we will augment the environment
+        vreps_env = reverse vreps_p ++ reverse vreps_np
+
+        -- new env and depth
+        vreps_env_tszsw = map (taggedSizeW.snd) vreps_env
+        p' = addListToFM p (zip (map fst vreps_env) 
+                                (mkStackOffsets d vreps_env_tszsw))
+        d' = d + sum vreps_env_tszsw
+
+        -- code to unpack the ptrs
+        ptrs_szw = sum (map (untaggedSizeW.snd) vreps_p)
+        code_p | null vreps_p = nilOL
+               | otherwise    = unitOL (UNPACK ptrs_szw)
+
+        -- code to unpack the nonptrs
+        vreps_env_uszw = sum (map (untaggedSizeW.snd) vreps_env)
+        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)
+           = case npr of
+                IntRep -> approved ; FloatRep -> approved
+                DoubleRep -> approved ; AddrRep -> approved
+                CharRep -> approved
+                _ -> pprPanic "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
+                usizeW   = untaggedSizeW npr
+                tsizeW   = taggedSizeW npr
+
 
 -- Push an atom onto the stack, returning suitable code & number of
 -- stack words used.  Pushes it either tagged or untagged, since 
@@ -490,21 +610,39 @@ mkUnpackCode off_h off_s (r:rs)
 -- 6 stack has valid words 0 .. 5.
 
 pushAtom :: Bool -> Int -> BCEnv -> AnnExpr' Id VarSet -> (BCInstrList, Int)
-pushAtom tagged d p (AnnVar v) 
-   = let str = "\npushAtom " ++ showSDocDebug (ppr v) ++ ", depth = " ++ show d
-               ++ ", env =\n" ++ 
-               showSDocDebug (nest 4 (vcat (map ppr (fmToList p))))
-               ++ " -->\n" ++
+pushAtom tagged d p (AnnVar v)
+
+   | idPrimRep v == VoidRep
+   = ASSERT(tagged)
+     (unitOL (PUSH_TAG 0), 1)
+
+   | Just primop <- isPrimOpId_maybe v
+   = case primop of
+        CCallOp _ -> panic "pushAtom: byte code generator can't handle CCalls"
+        other     -> (unitOL (PUSH_G (Right primop)), 1)
+
+   | otherwise
+   = let str = "\npushAtom " ++ showSDocDebug (ppr v) 
+               ++ " :: " ++ showSDocDebug (pprType (idType v))
+               ++ ", depth = " ++ show d
+               ++ ", tagged = " ++ show tagged ++ ", env =\n" ++ 
+               showSDocDebug (ppBCEnv p)
+               ++ " --> words: " ++ show (snd result) ++ "\n" ++
                showSDoc (nest 4 (vcat (map ppr (fromOL (fst result)))))
                ++ "\nendPushAtom " ++ showSDocDebug (ppr v)
+                  where
+                     cmp_snd x y = compare (snd x) (snd y)
          str' = if str == str then str else str
 
          result
             = case lookupBCEnv_maybe p v of
-                 Just d_v -> (toOL (nOfThem nwords (PUSH_L (d-d_v+sz_t-2))), sz_t)
-                 Nothing  -> ASSERT(sz_t == 1) (unitOL (PUSH_G nm), sz_t)
+                 Just d_v -> (toOL (nOfThem nwords (PUSH_L (d-d_v+sz_t-2))), nwords)
+                 Nothing  -> ASSERT(sz_t == 1) (unitOL (PUSH_G (Left nm)), nwords)
+
+         nm = case isDataConId_maybe v of
+                 Just c  -> getName c
+                 Nothing -> getName v
 
-         nm     = getName v
          sz_t   = taggedIdSizeW v
          sz_u   = untaggedIdSizeW v
          nwords = if tagged then sz_t else sz_u
@@ -518,22 +656,64 @@ pushAtom True d p (AnnLit lit)
 
 pushAtom False d p (AnnLit lit)
    = case lit of
+        MachWord w   -> code WordRep
         MachInt i    -> code IntRep
         MachFloat r  -> code FloatRep
         MachDouble r -> code DoubleRep
+        MachChar c   -> code CharRep
+        MachStr s    -> pushStr s
      where
         code rep
            = let size_host_words = untaggedSizeW rep
-                 size_in_word32s = (size_host_words * wORD_SIZE) `div` 4
-             in (unitOL (PUSH_UBX lit size_in_word32s), size_host_words)
+             in (unitOL (PUSH_UBX lit size_host_words), size_host_words)
+
+        pushStr s 
+           = let mallocvilleAddr
+                    = case s of
+                         CharStr s i -> A# s
+
+                         FastString _ l ba -> 
+                            -- sigh, a string in the heap is no good to us.
+                            -- We need a static C pointer, since the type of 
+                            -- a string literal is Addr#.  So, copy the string 
+                            -- into C land and introduce a memory leak 
+                            -- 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)
+                                      writeCharOffAddr (A# a#) n '\0'
+                                      return (A# a#)
+                                   )
+                         _ -> panic "StgInterp.lit2expr: unhandled string constant type"
+
+                 addrLit 
+                    = MachInt (toInteger (addrToInt mallocvilleAddr))
+             in
+                -- Get the addr on the stack, untaggedly
+                (unitOL (PUSH_UBX addrLit 1), 1)
+
+
+
+
 
 pushAtom tagged d p (AnnApp f (_, AnnType _))
    = pushAtom tagged d p (snd f)
 
+pushAtom tagged d p (AnnNote note e)
+   = pushAtom tagged d p (snd e)
+
+pushAtom tagged d p (AnnLam x e) 
+   | isTyVar x 
+   = pushAtom tagged d p (snd e)
+
 pushAtom tagged d p other
    = pprPanic "ByteCodeGen.pushAtom" 
               (pprCoreExpr (deAnnotate (undefined, other)))
 
+foreign import "strncpy" strncpy :: Ptr a -> ByteArray# -> CInt -> IO ()
+
 
 -- Given a bunch of alts code and their discrs, do the donkey work
 -- of making a multiway branch using a switch tree.
@@ -606,7 +786,7 @@ mkMultiBranch maybe_ncons raw_ways
 
          (algMinBound, algMaxBound)
             = case maybe_ncons of
-                 Just n  -> (fIRST_TAG, fIRST_TAG + n - 1)
+                 Just n  -> (0, n - 1)
                  Nothing -> (minBound, maxBound)
 
          (DiscrI i1) `eqAlt` (DiscrI i2) = i1 == i2
@@ -669,12 +849,12 @@ instance Outputable Discr where
 
 -- Find things in the BCEnv (the what's-on-the-stack-env)
 -- See comment preceding pushAtom for precise meaning of env contents
-lookupBCEnv :: BCEnv -> Id -> Int
-lookupBCEnv env nm
-   = case lookupFM env nm of
-        Nothing -> pprPanic "lookupBCEnv" 
-                            (ppr nm $$ char ' ' $$ vcat (map ppr (fmToList env)))
-        Just xx -> xx
+--lookupBCEnv :: BCEnv -> Id -> Int
+--lookupBCEnv env nm
+--   = case lookupFM env nm of
+--        Nothing -> pprPanic "lookupBCEnv" 
+--                            (ppr nm $$ char ' ' $$ vcat (map ppr (fmToList env)))
+--        Just xx -> xx
 
 lookupBCEnv_maybe :: BCEnv -> Id -> Maybe Int
 lookupBCEnv_maybe = lookupFM
@@ -698,6 +878,10 @@ taggedIdSizeW, untaggedIdSizeW :: Id -> Int
 taggedIdSizeW   = taggedSizeW   . typePrimRep . idType
 untaggedIdSizeW = untaggedSizeW . typePrimRep . idType
 
+unboxedTupleException :: a
+unboxedTupleException 
+   = throwDyn (Panic "bytecode generator can't handle unboxed tuples")
+
 \end{code}
 
 %************************************************************************
@@ -713,9 +897,6 @@ data BcM_State
 
 type BcM result = BcM_State -> (result, BcM_State)
 
-mkBcM_State :: [ProtoBCO Name] -> Int -> BcM_State
-mkBcM_State = BcM_State
-
 runBc :: BcM_State -> BcM () -> BcM_State
 runBc init_st m = case m init_st of { (r,st) -> st }
 
@@ -746,746 +927,3 @@ getLabelBc st
    = (nextlabel st, st{nextlabel = 1 + nextlabel st})
 
 \end{code}
-
-%************************************************************************
-%*                                                                     *
-\subsection{The bytecode assembler}
-%*                                                                     *
-%************************************************************************
-
-The object format for bytecodes is: 16 bits for the opcode, and 16 for
-each field -- so the code can be considered a sequence of 16-bit ints.
-Each field denotes either a stack offset or number of items on the
-stack (eg SLIDE), and index into the pointer table (eg PUSH_G), an
-index into the literal table (eg PUSH_I/D/L), or a bytecode address in
-this BCO.
-
-\begin{code}
--- Top level assembler fn.
-assembleBCO :: ProtoBCO Name -> IO UnlinkedBCO
-
-assembleBCO (ProtoBCO nm instrs origin)
-   = let
-         -- pass 1: collect up the offsets of the local labels
-         label_env = mkLabelEnv emptyFM 0 instrs
-
-         mkLabelEnv env i_offset [] = env
-         mkLabelEnv env i_offset (i:is)
-            = let new_env 
-                     = case i of LABEL n -> addToFM env n i_offset ; _ -> env
-              in  mkLabelEnv new_env (i_offset + instrSizeB i) is
-
-         findLabel lab
-            = case lookupFM label_env lab of
-                 Just bco_offset -> bco_offset
-                 Nothing -> pprPanic "assembleBCO.findLabel" (int lab)
-
-         init_n_insns = 10
-         init_n_lits  = 4
-         init_n_ptrs  = 4
-         init_n_itbls = 4
-     in
-     do  insns <- newXIOUArray init_n_insns :: IO (XIOUArray Word16)
-         lits  <- newXIOUArray init_n_lits  :: IO (XIOUArray Word32)
-         ptrs  <- newXIOArray  init_n_ptrs  -- :: IO (XIOArray Name)
-         itbls <- newXIOArray  init_n_itbls -- :: IO (XIOArray Name)
-
-         -- pass 2: generate the instruction, ptr and nonptr bits
-         let init_asm_state = (insns,lits,ptrs,itbls)
-         final_asm_state <- mkBits findLabel init_asm_state instrs         
-
-         -- unwrap the expandable arrays
-         let final_insns = stuffXIOU insns
-             final_lits  = stuffXIOU lits
-             final_ptrs  = stuffXIO  ptrs
-             final_itbls = stuffXIO  itbls
-
-         return (UnlinkedBCO nm
-                             (usedXIOU insns) final_insns 
-                             (usedXIOU lits)  final_lits 
-                             (usedXIO  ptrs)  final_ptrs 
-                             (usedXIO  itbls) final_itbls)
-
-
--- instrs nonptrs ptrs itbls
-type AsmState = (XIOUArray Word16, XIOUArray Word32, XIOArray Name, XIOArray Name)
-
-
--- This is where all the action is (pass 2 of the assembler)
-mkBits :: (Int -> Int)                         -- label finder
-       -> AsmState
-       -> [BCInstr]                    -- instructions (in)
-       -> IO AsmState
-
-mkBits findLabel st proto_insns
-  = foldM doInstr st proto_insns
-    where
-       doInstr :: AsmState -> BCInstr -> IO AsmState
-       doInstr st i
-          = case i of
-               ARGCHECK  n        -> instr2 st i_ARGCHECK n
-               PUSH_L    o1       -> instr2 st i_PUSH_L o1
-               PUSH_LL   o1 o2    -> instr3 st i_PUSH_LL o1 o2
-               PUSH_LLL  o1 o2 o3 -> instr4 st i_PUSH_LLL o1 o2 o3
-               PUSH_G    nm       -> do (p, st2) <- ptr st nm
-                                        instr2 st2 i_PUSH_G p
-               PUSH_AS   nm pk    -> do (p, st2)  <- ptr st nm
-                                        (np, st3) <- ret_itbl st2 pk
-                                        instr3 st3 i_PUSH_AS p np
-               PUSH_UBX lit nw32s -> do (np, st2) <- literal st lit
-                                        instr3 st2 i_PUSH_UBX np nw32s
-               PUSH_TAG  tag      -> instr2 st i_PUSH_TAG tag
-               SLIDE     n by     -> instr3 st i_SLIDE n by
-               ALLOC     n        -> instr2 st i_ALLOC n
-               MKAP      off sz   -> instr3 st i_MKAP off sz
-               UNPACK    n        -> instr2 st i_UNPACK n
-               UPK_TAG   n m k    -> instr4 st i_UPK_TAG n m k
-               PACK      dcon sz  -> do (itbl_no,st2) <- itbl st dcon
-                                        instr3 st2 i_PACK itbl_no sz
-               LABEL     lab      -> return st
-               TESTLT_I  i l      -> do (np, st2) <- int st i
-                                        instr3 st2 i_TESTLT_I np (findLabel l)
-               TESTEQ_I  i l      -> do (np, st2) <- int st i
-                                        instr3 st2 i_TESTEQ_I np (findLabel l)
-               TESTLT_F  f l      -> do (np, st2) <- float st f
-                                        instr3 st2 i_TESTLT_F np (findLabel l)
-               TESTEQ_F  f l      -> do (np, st2) <- float st f
-                                        instr3 st2 i_TESTEQ_F np (findLabel l)
-               TESTLT_D  d l      -> do (np, st2) <- double st d
-                                        instr3 st2 i_TESTLT_D np (findLabel l)
-               TESTEQ_D  d l      -> do (np, st2) <- double st d
-                                        instr3 st2 i_TESTEQ_D np (findLabel l)
-               TESTLT_P  i l      -> do (np, st2) <- int st i
-                                        instr3 st2 i_TESTLT_P np (findLabel l)
-               TESTEQ_P  i l      -> do (np, st2) <- int st i
-                                        instr3 st2 i_TESTEQ_P np (findLabel l)
-               CASEFAIL           -> instr1 st i_CASEFAIL
-               ENTER              -> instr1 st i_ENTER
-               RETURN             -> instr1 st i_RETURN
-
-       i2s :: Int -> Word16
-       i2s = fromIntegral
-
-       instr1 (st_i0,st_l0,st_p0,st_I0) i1
-          = do st_i1 <- addToXIOUArray st_i0 (i2s i1)
-               return (st_i1,st_l0,st_p0,st_I0)
-
-       instr2 (st_i0,st_l0,st_p0,st_I0) i1 i2
-          = do st_i1 <- addToXIOUArray st_i0 (i2s i1)
-               st_i2 <- addToXIOUArray st_i1 (i2s i2)
-               return (st_i2,st_l0,st_p0,st_I0)
-
-       instr3 (st_i0,st_l0,st_p0,st_I0) i1 i2 i3
-          = do st_i1 <- addToXIOUArray st_i0 (i2s i1)
-               st_i2 <- addToXIOUArray st_i1 (i2s i2)
-               st_i3 <- addToXIOUArray st_i2 (i2s i3)
-               return (st_i3,st_l0,st_p0,st_I0)
-
-       instr4 (st_i0,st_l0,st_p0,st_I0) i1 i2 i3 i4
-          = do st_i1 <- addToXIOUArray st_i0 (i2s i1)
-               st_i2 <- addToXIOUArray st_i1 (i2s i2)
-               st_i3 <- addToXIOUArray st_i2 (i2s i3)
-               st_i4 <- addToXIOUArray st_i3 (i2s i4)
-               return (st_i4,st_l0,st_p0,st_I0)
-
-       float (st_i0,st_l0,st_p0,st_I0) f
-          = do let w32s = mkLitF f
-               st_l1 <- addListToXIOUArray st_l0 w32s
-               return (usedXIOU st_l0, (st_i0,st_l1,st_p0,st_I0))
-
-       double (st_i0,st_l0,st_p0,st_I0) d
-          = do let w32s = mkLitD d
-               st_l1 <- addListToXIOUArray st_l0 w32s
-               return (usedXIOU st_l0, (st_i0,st_l1,st_p0,st_I0))
-
-       int (st_i0,st_l0,st_p0,st_I0) i
-          = do let w32s = mkLitI i
-               st_l1 <- addListToXIOUArray st_l0 w32s
-               return (usedXIOU st_l0, (st_i0,st_l1,st_p0,st_I0))
-
-       addr (st_i0,st_l0,st_p0,st_I0) a
-          = do let w32s = mkLitA a
-               st_l1 <- addListToXIOUArray st_l0 w32s
-               return (usedXIOU st_l0, (st_i0,st_l1,st_p0,st_I0))
-
-       ptr (st_i0,st_l0,st_p0,st_I0) p
-          = do st_p1 <- addToXIOArray st_p0 p
-               return (usedXIO st_p0, (st_i0,st_l0,st_p1,st_I0))
-
-       itbl (st_i0,st_l0,st_p0,st_I0) dcon
-          = do st_I1 <- addToXIOArray st_I0 (getName dcon)
-               return (usedXIO st_I0, (st_i0,st_l0,st_p0,st_I1))
-
-       literal st (MachInt j)    = int st (fromIntegral j)
-       literal st (MachFloat r)  = float st (fromRational r)
-       literal st (MachDouble r) = double st (fromRational r)
-
-       ret_itbl st pk
-          = addr st ret_itbl_addr
-            where
-               ret_itbl_addr 
-                  = case pk of
-                       IntRep    -> stg_ctoi_ret_R1_info
-                       FloatRep  -> stg_ctoi_ret_F1_info
-                       DoubleRep -> stg_ctoi_ret_D1_info
-                    where  -- TEMP HACK
-                       stg_ctoi_ret_F1_info = nullAddr
-                       stg_ctoi_ret_D1_info = nullAddr
-                     
-foreign label "stg_ctoi_ret_R1_info" stg_ctoi_ret_R1_info :: Addr
---foreign label "stg_ctoi_ret_F1_info" stg_ctoi_ret_F1_info :: Addr
---foreign label "stg_ctoi_ret_D1_info" stg_ctoi_ret_D1_info :: Addr
-
--- The size in bytes of an instruction.
-instrSizeB :: BCInstr -> Int
-instrSizeB instr
-   = case instr of
-        ARGCHECK _     -> 4
-        PUSH_L   _     -> 4
-        PUSH_LL  _ _   -> 6
-        PUSH_LLL _ _ _ -> 8
-        PUSH_G   _     -> 4
-        SLIDE    _ _   -> 6
-        ALLOC    _     -> 4
-        MKAP     _ _   -> 6
-        UNPACK   _     -> 4
-        PACK     _ _   -> 6
-        LABEL    _     -> 4
-        TESTLT_I _ _   -> 6
-        TESTEQ_I _ _   -> 6
-        TESTLT_F _ _   -> 6
-        TESTEQ_F _ _   -> 6
-        TESTLT_D _ _   -> 6
-        TESTEQ_D _ _   -> 6
-        TESTLT_P _ _   -> 6
-        TESTEQ_P _ _   -> 6
-        CASEFAIL       -> 2
-        ENTER          -> 2
-        RETURN         -> 2
-
-
--- Sizes of Int, Float and Double literals, in units of 32-bitses
-intLitSz32s, floatLitSz32s, doubleLitSz32s, addrLitSz32s :: Int
-intLitSz32s    = wORD_SIZE `div` 4
-floatLitSz32s  = 1     -- Assume IEEE floats
-doubleLitSz32s = 2
-addrLitSz32s   = intLitSz32s
-
--- Make lists of 32-bit words for literals, so that when the
--- words are placed in memory at increasing addresses, the
--- bit pattern is correct for the host's word size and endianness.
-mkLitI :: Int    -> [Word32]
-mkLitF :: Float  -> [Word32]
-mkLitD :: Double -> [Word32]
-mkLitA :: Addr   -> [Word32]
-
-mkLitF f
-   = runST (do
-        arr <- newFloatArray ((0::Int),0)
-        writeFloatArray arr 0 f
-        f_arr <- castSTUArray arr
-        w0 <- readWord32Array f_arr 0
-        return [w0]
-     )
-
-mkLitD d
-   = runST (do
-        arr <- newDoubleArray ((0::Int),0)
-        writeDoubleArray arr 0 d
-        d_arr <- castSTUArray arr
-        w0 <- readWord32Array d_arr 0
-        w1 <- readWord32Array d_arr 1
-        return [w0,w1]
-     )
-
-mkLitI i
-   | wORD_SIZE == 4
-   = runST (do
-        arr <- newIntArray ((0::Int),0)
-        writeIntArray arr 0 i
-        i_arr <- castSTUArray arr
-        w0 <- readWord32Array i_arr 0
-        return [w0]
-     )
-   | wORD_SIZE == 8
-   = runST (do
-        arr <- newIntArray ((0::Int),0)
-        writeIntArray arr 0 i
-        i_arr <- castSTUArray arr
-        w0 <- readWord32Array i_arr 0
-        w1 <- readWord32Array i_arr 1
-        return [w0,w1]
-     )
-   
-mkLitA a
-   | wORD_SIZE == 4
-   = runST (do
-        arr <- newAddrArray ((0::Int),0)
-        writeAddrArray arr 0 a
-        a_arr <- castSTUArray arr
-        w0 <- readWord32Array a_arr 0
-        return [w0]
-     )
-   | wORD_SIZE == 8
-   = runST (do
-        arr <- newAddrArray ((0::Int),0)
-        writeAddrArray arr 0 a
-        a_arr <- castSTUArray arr
-        w0 <- readWord32Array a_arr 0
-        w1 <- readWord32Array a_arr 1
-        return [w0,w1]
-     )
-   
-
-
--- Zero-based expandable arrays
-data XIOUArray ele 
-   = XIOUArray { usedXIOU :: Int, stuffXIOU :: (IOUArray Int ele) }
-data XIOArray ele 
-   = XIOArray { usedXIO :: Int , stuffXIO :: (IOArray Int ele) }
-
-newXIOUArray size
-   = do arr <- newArray (0, size-1)
-        return (XIOUArray 0 arr)
-
-addListToXIOUArray xarr []
-   = return xarr
-addListToXIOUArray xarr (x:xs)
-   = addToXIOUArray xarr x >>= \ xarr' -> addListToXIOUArray xarr' xs
-
-
-addToXIOUArray :: MArray IOUArray a IO
-                  => XIOUArray a -> a -> IO (XIOUArray a)
-addToXIOUArray (XIOUArray n_arr arr) x
-   = case bounds arr of
-        (lo, hi) -> ASSERT(lo == 0)
-                    if   n_arr > hi
-                    then do new_arr <- newArray (0, 2*hi-1)
-                            copy hi arr new_arr
-                            addToXIOUArray (XIOUArray n_arr new_arr) x
-                    else do writeArray arr n_arr x
-                            return (XIOUArray (n_arr+1) arr)
-     where
-        copy :: MArray IOUArray a IO
-                => Int -> IOUArray Int a -> IOUArray Int a -> IO ()
-        copy n src dst
-           | n < 0     = return ()
-           | otherwise = do nx <- readArray src n
-                            writeArray dst n nx
-                            copy (n-1) src dst
-
-
-
-newXIOArray size
-   = do arr <- newArray (0, size-1)
-        return (XIOArray 0 arr)
-
-addToXIOArray :: XIOArray a -> a -> IO (XIOArray a)
-addToXIOArray (XIOArray n_arr arr) x
-   = case bounds arr of
-        (lo, hi) -> ASSERT(lo == 0)
-                    if   n_arr > hi
-                    then do new_arr <- newArray (0, 2*hi-1)
-                            copy hi arr new_arr
-                            addToXIOArray (XIOArray n_arr new_arr) x
-                    else do writeArray arr n_arr x
-                            return (XIOArray (n_arr+1) arr)
-     where
-        copy :: Int -> IOArray Int a -> IOArray Int a -> IO ()
-        copy n src dst
-           | n < 0     = return ()
-           | otherwise = do nx <- readArray src n
-                            writeArray dst n nx
-                            copy (n-1) src dst
-
-\end{code}
-
-%************************************************************************
-%*                                                                     *
-\subsection{Linking interpretables into something we can run}
-%*                                                                     *
-%************************************************************************
-
-\begin{code}
-
-{- 
-data UnlinkedBCO
-   = UnlinkedBCO Int (IOUArray Int Word16)     -- #insns insns
-                 Int (IOUArray Int Word32)     -- #literals literals
-                 Int (IOArray Int Name)                -- #ptrs ptrs
-                 Int (IOArray Int Name)                -- #itblrefs itblrefs
-
-data BCO# = BCO# ByteArray#            -- instrs   :: array Word16#
-                 ByteArray#            -- literals :: array Word32#
-                 PtrArray#             -- ptrs     :: Array HValue
-                 ByteArray#            -- itbls    :: Array Addr#
--}
-
-data LinkedBCO = LinkedBCO BCO#
-
-
-
-GLOBAL_VAR(v_cafTable, [], [HValue])
-
-addCAF :: HValue -> IO ()
-addCAF x = do xs <- readIORef v_cafTable; writeIORef v_cafTable (x:xs)
-
-linkIModules :: ItblEnv    -- incoming global itbl env; returned updated
-            -> ClosureEnv -- incoming global closure env; returned updated
-            -> [([UnlinkedBCO], ItblEnv)]
-            -> IO ([HValue], ItblEnv, ClosureEnv)
-linkIModules gie gce mods = do
-  let (bcoss, ies) = unzip mods
-      bcos = concat bcoss
-      top_level_binders = map nameOfUnlinkedBCO bcos
-      final_gie = foldr plusFM gie ies
-  
-  (new_bcos, new_gce) <-
-    fixIO (\ ~(new_bcos, new_gce) -> do
-
-      new_bcos <- linkBCOs final_gie new_gce bcos
-
-      let new_gce = addListToFM gce (zip top_level_binders new_bcos)
-
-      return (new_bcos, new_gce))
-
-  return (new_bcos, final_gie, new_gce)
-
-
-
-linkBCOs :: ItblEnv -> ClosureEnv -> [UnlinkedBCO] 
-         -> IO [HValue]   -- IO [BCO#] really
-linkBCOs ie ce binds = mapM (linkBCO ie ce) binds
-
-linkBCO ie ce (UnlinkedBCO nm 
-                           n_insns insns n_literals literals 
-                           n_ptrs ptrs n_itbls itbls)
-   = do linked_ptrs <- mapArray (lookupCE ce) ptrs
-        linked_itbls <- mapArray (lookupIE ie) itbls
-
-        ptrs_froz <- freeze linked_ptrs
-        let ptrs_parr = case ptrs_froz of Array lo hi parr -> parr
-
-        insns_froz <- freeze insns
-        let insns_barr = case insns_froz of UArray lo hi barr -> barr
-
-        literals_froz <- freeze literals
-        let literals_barr = case literals_froz of UArray lo hi barr -> barr
-
-        itbls_froz <- freeze linked_itbls
-        let itbls_barr = case itbls_froz of UArray lo hi barr -> barr
-
-        BCO bco# <- newBCO insns_barr literals_barr ptrs_parr itbls_barr
-     
-        return (unsafeCoerce# bco#)
-
-data BCO = BCO BCO#
-
-newBCO :: ByteArray# -> ByteArray# -> Array# a -> ByteArray# -> IO BCO
-newBCO a b c d = IO (\s -> case newBCO# a b c d s of (# s1, bco #) -> (# s1, BCO bco #))
-
-
-lookupCE :: ClosureEnv -> Name -> HValue
-lookupCE ce nm 
-   = case lookupFM ce nm of
-        Just aa -> unsafeCoerce# aa
-        Nothing -> pprPanic "ByteCodeGen.lookupCE" (ppr nm)
-
-lookupIE :: ItblEnv -> Name -> Addr
-lookupIE ie nm 
-   = case lookupFM ie nm of
-        Just (Ptr a) -> a
-        Nothing      -> pprPanic "ByteCodeGen.lookupIE" (ppr nm)
-
-
-
-{-
-lookupCon ie con = 
-  case lookupFM ie con of
-    Just (Ptr addr) -> return addr
-    Nothing   -> do
-       -- try looking up in the object files.
-        m <- lookupSymbol (nameToCLabel con "con_info")
-       case m of
-           Just addr -> return addr
-           Nothing   -> pprPanic "linkIExpr" (ppr con)
-
--- nullary constructors don't have normal _con_info tables.
-lookupNullaryCon ie con =
-  case lookupFM ie con of
-    Just (Ptr addr) -> return (ConApp addr)
-    Nothing -> do
-       -- try looking up in the object files.
-       m <- lookupSymbol (nameToCLabel con "closure")
-       case m of
-           Just (A# addr) -> return (Native (unsafeCoerce# addr))
-           Nothing   -> pprPanic "lookupNullaryCon" (ppr con)
-
-
-lookupNative ce var =
-  unsafeInterleaveIO (do
-      case lookupFM ce var of
-       Just e  -> return (Native e)
-       Nothing -> do
-           -- try looking up in the object files.
-           let lbl = (nameToCLabel var "closure")
-           m <- lookupSymbol lbl
-           case m of
-               Just (A# addr)
-                   -> do addCAF (unsafeCoerce# addr)
-                         return (Native (unsafeCoerce# addr))
-               Nothing   -> pprPanic "linkIExpr" (ppr var)
-  )
-
--- some VarI/VarP refer to top-level interpreted functions; we change
--- them into Natives here.
-lookupVar ce f v =
-  unsafeInterleaveIO (
-       case lookupFM ce (getName v) of
-           Nothing -> return (f v)
-           Just e  -> return (Native e)
-  )
-
--- HACK!!!  ToDo: cleaner
-nameToCLabel :: Name -> String{-suffix-} -> String
-nameToCLabel n suffix =
-  _UNPK_(moduleNameFS (rdrNameModule rn)) 
-  ++ '_':occNameString(rdrNameOcc rn) ++ '_':suffix
-  where rn = toRdrName n
--}
-\end{code}
-
-%************************************************************************
-%*                                                                     *
-\subsection{Manufacturing of info tables for DataCons}
-%*                                                                     *
-%************************************************************************
-
-\begin{code}
-
-#if __GLASGOW_HASKELL__ <= 408
-type ItblPtr = Addr
-#else
-type ItblPtr = Ptr StgInfoTable
-#endif
-
--- Make info tables for the data decls in this module
-mkITbls :: [TyCon] -> IO ItblEnv
-mkITbls [] = return emptyFM
-mkITbls (tc:tcs) = do itbls  <- mkITbl tc
-                      itbls2 <- mkITbls tcs
-                      return (itbls `plusFM` itbls2)
-
-mkITbl :: TyCon -> IO ItblEnv
-mkITbl tc
---   | trace ("TYCON: " ++ showSDoc (ppr tc)) False
---   = error "?!?!"
-   | not (isDataTyCon tc) 
-   = return emptyFM
-   | n == length dcs  -- paranoia; this is an assertion.
-   = make_constr_itbls dcs
-     where
-        dcs = tyConDataCons tc
-        n   = tyConFamilySize tc
-
-cONSTR :: Int
-cONSTR = 1  -- as defined in ghc/includes/ClosureTypes.h
-
--- Assumes constructors are numbered from zero, not one
-make_constr_itbls :: [DataCon] -> IO ItblEnv
-make_constr_itbls cons
-   | length cons <= 8
-   = do is <- mapM mk_vecret_itbl (zip cons [0..])
-       return (listToFM is)
-   | otherwise
-   = do is <- mapM mk_dirret_itbl (zip cons [0..])
-       return (listToFM is)
-     where
-        mk_vecret_itbl (dcon, conNo)
-           = mk_itbl dcon conNo (vecret_entry conNo)
-        mk_dirret_itbl (dcon, conNo)
-           = mk_itbl dcon conNo stg_interp_constr_entry
-
-        mk_itbl :: DataCon -> Int -> Addr -> IO (Name,ItblPtr)
-        mk_itbl dcon conNo entry_addr
-           = let (tot_wds, ptr_wds, _) 
-                    = mkVirtHeapOffsets typePrimRep (dataConRepArgTys dcon)
-                 ptrs = ptr_wds
-                 nptrs  = tot_wds - ptr_wds
-                 itbl  = StgInfoTable {
-                           ptrs = fromIntegral ptrs, nptrs = fromIntegral nptrs,
-                           tipe = fromIntegral cONSTR,
-                           srtlen = fromIntegral conNo,
-                           code0 = fromIntegral code0, code1 = fromIntegral code1,
-                           code2 = fromIntegral code2, code3 = fromIntegral code3,
-                           code4 = fromIntegral code4, code5 = fromIntegral code5,
-                           code6 = fromIntegral code6, code7 = fromIntegral code7 
-                        }
-                 -- Make a piece of code to jump to "entry_label".
-                 -- This is the only arch-dependent bit.
-                 -- On x86, if entry_label has an address 0xWWXXYYZZ,
-                 -- emit   movl $0xWWXXYYZZ,%eax  ;  jmp *%eax
-                 -- which is
-                 -- B8 ZZ YY XX WW FF E0
-                 (code0,code1,code2,code3,code4,code5,code6,code7)
-                    = (0xB8, byte 0 entry_addr_w, byte 1 entry_addr_w, 
-                             byte 2 entry_addr_w, byte 3 entry_addr_w, 
-                       0xFF, 0xE0, 
-                       0x90 {-nop-})
-
-                 entry_addr_w :: Word32
-                 entry_addr_w = fromIntegral (addrToInt entry_addr)
-             in
-                 do addr <- malloc
-                    --putStrLn ("SIZE of itbl is " ++ show (sizeOf itbl))
-                    --putStrLn ("# ptrs  of itbl is " ++ show ptrs)
-                    --putStrLn ("# nptrs of itbl is " ++ show nptrs)
-                    poke addr itbl
-                    return (getName dcon, addr `plusPtr` 8)
-
-
-byte :: Int -> Word32 -> Word32
-byte 0 w = w .&. 0xFF
-byte 1 w = (w `shiftR` 8) .&. 0xFF
-byte 2 w = (w `shiftR` 16) .&. 0xFF
-byte 3 w = (w `shiftR` 24) .&. 0xFF
-
-
-vecret_entry 0 = stg_interp_constr1_entry
-vecret_entry 1 = stg_interp_constr2_entry
-vecret_entry 2 = stg_interp_constr3_entry
-vecret_entry 3 = stg_interp_constr4_entry
-vecret_entry 4 = stg_interp_constr5_entry
-vecret_entry 5 = stg_interp_constr6_entry
-vecret_entry 6 = stg_interp_constr7_entry
-vecret_entry 7 = stg_interp_constr8_entry
-
--- entry point for direct returns for created constr itbls
-foreign label "stg_interp_constr_entry" stg_interp_constr_entry :: Addr
--- and the 8 vectored ones
-foreign label "stg_interp_constr1_entry" stg_interp_constr1_entry :: Addr
-foreign label "stg_interp_constr2_entry" stg_interp_constr2_entry :: Addr
-foreign label "stg_interp_constr3_entry" stg_interp_constr3_entry :: Addr
-foreign label "stg_interp_constr4_entry" stg_interp_constr4_entry :: Addr
-foreign label "stg_interp_constr5_entry" stg_interp_constr5_entry :: Addr
-foreign label "stg_interp_constr6_entry" stg_interp_constr6_entry :: Addr
-foreign label "stg_interp_constr7_entry" stg_interp_constr7_entry :: Addr
-foreign label "stg_interp_constr8_entry" stg_interp_constr8_entry :: Addr
-
-
-
-data Constructor = Constructor Int{-ptrs-} Int{-nptrs-}
-
-
--- Ultra-minimalist version specially for constructors
-data StgInfoTable = StgInfoTable {
-   ptrs :: Word16,
-   nptrs :: Word16,
-   srtlen :: Word16,
-   tipe :: Word16,
-   code0, code1, code2, code3, code4, code5, code6, code7 :: Word8
-}
-
-
-instance Storable StgInfoTable where
-
-   sizeOf itbl 
-      = (sum . map (\f -> f itbl))
-        [fieldSz ptrs, fieldSz nptrs, fieldSz srtlen, fieldSz tipe,
-         fieldSz code0, fieldSz code1, fieldSz code2, fieldSz code3, 
-         fieldSz code4, fieldSz code5, fieldSz code6, fieldSz code7]
-
-   alignment itbl 
-      = (sum . map (\f -> f itbl))
-        [fieldAl ptrs, fieldAl nptrs, fieldAl srtlen, fieldAl tipe,
-         fieldAl code0, fieldAl code1, fieldAl code2, fieldAl code3, 
-         fieldAl code4, fieldAl code5, fieldAl code6, fieldAl code7]
-
-   poke a0 itbl
-      = do a1 <- store (ptrs   itbl) (castPtr a0)
-           a2 <- store (nptrs  itbl) a1
-           a3 <- store (tipe   itbl) a2
-           a4 <- store (srtlen itbl) a3
-           a5 <- store (code0  itbl) a4
-           a6 <- store (code1  itbl) a5
-           a7 <- store (code2  itbl) a6
-           a8 <- store (code3  itbl) a7
-           a9 <- store (code4  itbl) a8
-           aA <- store (code5  itbl) a9
-           aB <- store (code6  itbl) aA
-           aC <- store (code7  itbl) aB
-           return ()
-
-   peek a0
-      = do (a1,ptrs)   <- load (castPtr a0)
-           (a2,nptrs)  <- load a1
-           (a3,tipe)   <- load a2
-           (a4,srtlen) <- load a3
-           (a5,code0)  <- load a4
-           (a6,code1)  <- load a5
-           (a7,code2)  <- load a6
-           (a8,code3)  <- load a7
-           (a9,code4)  <- load a8
-           (aA,code5)  <- load a9
-           (aB,code6)  <- load aA
-           (aC,code7)  <- load aB
-           return StgInfoTable { ptrs = ptrs, nptrs = nptrs, 
-                                 srtlen = srtlen, tipe = tipe,
-                                 code0 = code0, code1 = code1, code2 = code2,
-                                 code3 = code3, code4 = code4, code5 = code5,
-                                 code6 = code6, code7 = code7 }
-
-fieldSz :: (Storable a, Storable b) => (a -> b) -> a -> Int
-fieldSz sel x = sizeOf (sel x)
-
-fieldAl :: (Storable a, Storable b) => (a -> b) -> a -> Int
-fieldAl sel x = alignment (sel x)
-
-store :: Storable a => a -> Ptr a -> IO (Ptr b)
-store x addr = do poke addr x
-                  return (castPtr (addr `plusPtr` sizeOf x))
-
-load :: Storable a => Ptr a -> IO (Ptr b, a)
-load addr = do x <- peek addr
-               return (castPtr (addr `plusPtr` sizeOf x), x)
-
-\end{code}
-
-%************************************************************************
-%*                                                                     *
-\subsection{Connect to actual values for bytecode opcodes}
-%*                                                                     *
-%************************************************************************
-
-\begin{code}
-
-#include "Bytecodes.h"
-
-i_ARGCHECK = (bci_ARGCHECK :: Int)
-i_PUSH_L   = (bci_PUSH_L :: Int)
-i_PUSH_LL  = (bci_PUSH_LL :: Int)
-i_PUSH_LLL = (bci_PUSH_LLL :: Int)
-i_PUSH_G   = (bci_PUSH_G :: Int)
-i_PUSH_AS  = (bci_PUSH_AS :: Int)
-i_PUSH_UBX = (bci_PUSH_UBX :: Int)
-i_PUSH_TAG = (bci_PUSH_TAG :: Int)
-i_SLIDE    = (bci_SLIDE :: Int)
-i_ALLOC    = (bci_ALLOC :: Int)
-i_MKAP     = (bci_MKAP :: Int)
-i_UNPACK   = (bci_UNPACK :: Int)
-i_UPK_TAG  = (bci_UPK_TAG :: Int)
-i_PACK     = (bci_PACK :: Int)
-i_LABEL    = (bci_LABEL :: Int)
-i_TESTLT_I = (bci_TESTLT_I :: Int)
-i_TESTEQ_I = (bci_TESTEQ_I :: Int)
-i_TESTLT_F = (bci_TESTLT_F :: Int)
-i_TESTEQ_F = (bci_TESTEQ_F :: Int)
-i_TESTLT_D = (bci_TESTLT_D :: Int)
-i_TESTEQ_D = (bci_TESTEQ_D :: Int)
-i_TESTLT_P = (bci_TESTLT_P :: Int)
-i_TESTEQ_P = (bci_TESTEQ_P :: Int)
-i_CASEFAIL = (bci_CASEFAIL :: Int)
-i_ENTER    = (bci_ENTER :: Int)
-i_RETURN   = (bci_RETURN :: Int)
-
-\end{code}