Skip to content

Commit

Permalink
lib: add heap_path_not_Nil to Heap_List
Browse files Browse the repository at this point in the history
Signed-off-by: Michael McInerney <michael.mcinerney@proofcraft.systems>
  • Loading branch information
michaelmcinerney committed Feb 11, 2025
1 parent 0cba8a6 commit 2cc6de9
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions lib/Heap_List.thy
Original file line number Diff line number Diff line change
Expand Up @@ -53,6 +53,10 @@ lemma heap_path_None[simp]:
"heap_path hp None xs end = (xs = [] \<and> end = None)"
by (cases xs, auto)

lemma heap_path_not_Nil:
"heap_ls hp (Some st) ls \<Longrightarrow> ls \<noteq> []"
by fastforce

lemma heap_ls_unique:
"\<lbrakk> heap_ls hp x xs; heap_ls hp x ys \<rbrakk> \<Longrightarrow> xs = ys"
by (induct xs arbitrary: ys x; simp) (case_tac ys; clarsimp)
Expand Down

0 comments on commit 2cc6de9

Please sign in to comment.