Abstract
This Isabelle/HOL formalization builds on the
VeriComp entry of the Archive of Formal
Proofs to provide the following contributions:
- an operational semantics for a realistic virtual machine (Std) for dynamically typed programming languages;
- the formalization of an inline caching optimization (Inca), a proof of bisimulation with (Std), and a compilation function;
- the formalization of an unboxing optimization (Ubx), a proof of bisimulation with (Inca), and a simple compilation function.
License
History
- June 25, 2021
- proved conditional completeness of compilation
- June 14, 2021
- refactored function definitions to contain explicit basic blocks
Topics
Session Interpreter_Optimizations
- Env
- Env_list
- List_util
- Result
- Option_Extra
- Map_Extra
- AList_Extra
- Global
- Op
- OpInl
- Dynamic
- Inca
- Unboxed
- OpUbx
- Ubx
- Ubx_Verification
- Unboxed_lemmas
- Inca_to_Ubx_simulation
- Inca_Verification
- Inca_to_Ubx_compiler
- Op_example
- Std
- Std_to_Inca_simulation
- Std_to_Inca_compiler