lh-l4v/proof/refine/ARM/Invocations_R.thy

31 lines
776 B
Plaintext
Raw Normal View History

2014-07-14 19:32:44 +00:00
(*
* Copyright 2014, General Dynamics C4 Systems
*
* This software may be distributed and modified according to the terms of
* the GNU General Public License version 2. Note that NO WARRANTY is provided.
* See "LICENSE_GPLv2.txt" for details.
*
* @TAG(GD_GPL)
*)
theory Invocations_R
imports Invariants_H
begin
2019-11-27 02:57:28 +00:00
context begin interpretation Arch . (*FIXME: arch_split*)
2019-11-27 02:57:28 +00:00
lemma invocationType_eq[simp]:
2014-07-14 19:32:44 +00:00
"invocationType = invocation_type"
2019-11-27 02:57:28 +00:00
unfolding invocationType_def invocation_type_def Let_def
by (rule ext, simp) (metis from_to_enum maxBound_is_bound')
lemma genInvocationType_eq[simp]:
"genInvocationType = gen_invocation_type"
by (rule ext) (simp add: genInvocationType_def gen_invocation_type_def)
end
2019-11-27 02:57:28 +00:00
2014-07-14 19:32:44 +00:00
declare resolveAddressBits.simps[simp del]
end