Skip to content

Commit

Permalink
x64 crefine: remove unused lemmas
Browse files Browse the repository at this point in the history
Signed-off-by: Gerwin Klein <[email protected]>
  • Loading branch information
lsf37 committed Oct 23, 2024
1 parent bba80e3 commit 6febd3d
Showing 1 changed file with 0 additions and 15 deletions.
15 changes: 0 additions & 15 deletions proof/crefine/X64/Arch_C.thy
Original file line number Diff line number Diff line change
Expand Up @@ -1468,21 +1468,6 @@ lemma obj_at_pte_aligned:
elim!: is_aligned_weaken)
done

(* FIXME x64: dont know what these are for yet *)
lemma addrFromPPtr_mask_5:
"addrFromPPtr ptr && mask (5::nat) = ptr && mask (5::nat)"
apply (simp add:addrFromPPtr_def X64.pptrBase_def)
apply word_bitwise
apply (simp add:mask_def)
done

lemma addrFromPPtr_mask_6:
"addrFromPPtr ptr && mask (6::nat) = ptr && mask (6::nat)"
apply (simp add:addrFromPPtr_def X64.pptrBase_def)
apply word_bitwise
apply (simp add:mask_def)
done

lemma cpde_relation_invalid:
"cpde_relation pdea pde \<Longrightarrow> (pde_get_tag pde = scast pde_pde_pt \<and> pde_pde_pt_CL.present_CL (pde_pde_pt_lift pde) = 0) = isInvalidPDE pdea"
apply (simp add: cpde_relation_def Let_def)
Expand Down

0 comments on commit 6febd3d

Please sign in to comment.