Module Vmbytegen

val compile : fail_on_error:bool -> ?⁠universes:int -> Environ.env -> Constr.constr -> (Vmbytecodes.bytecodes * Vmbytecodes.bytecodes * Vmbytecodes.fv) option

Should only be used for monomorphic terms

init, fun, fv

val compile_constant_body : fail_on_error:bool -> Environ.env -> Declarations.universes -> (Constr.t Mod_subst.substituted'opaque) Declarations.constant_def -> Vmemitcodes.body_code option
val compile_alias : Names.Constant.t -> Vmemitcodes.body_code
val dump_bytecode : bool Stdlib.ref

Dump the bytecode after compilation (for debugging purposes)