aarch64 refine: lemma moved to Word_Lib

Signed-off-by: Gerwin Klein <gerwin.klein@proofcraft.systems>
This commit is contained in:
Gerwin Klein 2023-08-24 11:24:00 +02:00
parent fe3ebf03b9
commit dc4955de6e
No known key found for this signature in database
GPG Key ID: 20A847CE6AB7F5F3
1 changed files with 0 additions and 10 deletions

View File

@ -3503,16 +3503,6 @@ lemma createObjects_orig_cte_wp_at':
apply clarsimp
done
(* FIXME AARCH64 move to Word_Lib: shifting right by a bigger amount yields a smaller number *)
lemma le_shiftr_n:
fixes w :: "'a::len word"
shows "m \<le> n \<Longrightarrow> w >> n \<le> w >> m"
apply (unfold shiftr_def)
apply transfer
apply (simp add: take_bit_drop_bit)
apply (simp add: drop_bit_eq_div zdiv_mono2)
done
lemma createNewCaps_cte_wp_at':
"\<lbrace>\<lambda>s. cte_wp_at' P p s
\<and> range_cover ptr sz (APIType_capBits ty us) n \<and> n \<noteq> 0