Theory Sparc_State
section ‹SPARC V8 state model›
theory Sparc_State
imports Main Sparc_Types "../lib/wp/DetMonadLemmas" MMU
begin
section ‹state as a function›
record cpu_cache =
dcache:: cache_context
icache:: cache_context
text‹
The state @{term sparc_state} is defined as a tuple @{term cpu_context},
@{term user_context}, @{term mem_context}, defining the state of the CPU registers,
user registers, memory, cache, and delayed write pool respectively.
Additionally, a boolean indicates whether the state is
undefined or not.
›