Theory Word_Mem_Encoding_ARM_HYP
theory Word_Mem_Encoding_ARM_HYP
imports "../Vanilla32_Preliminaries"
begin
if_architecture_context (ARM_HYP)
begin
definition
word_tag :: "'a::len8 word itself ⇒ 'a word xtyp_info"
where
"word_tag (w::'a::len8 word itself) ≡
TypDesc (len_exp TYPE('a)) (TypScalar (len_of TYPE('a) div 8) (len_exp TYPE('a))
⦇field_access = λv bs. (rev o word_rsplit) v,
field_update = λbs v. (word_rcat (rev (take (len_of TYPE('a) div 8) bs))::'a::len8 word),
field_sz = (len_of TYPE('a) div 8)⦈)
(''word'' @ nat_to_bin_string (len_of TYPE('a)) )"
end
end