Skip to content
Snippets Groups Projects
Commit 63f6c55b authored by Robbert Krebbers's avatar Robbert Krebbers
Browse files

Test `iInduction` with multiple IHs in the tree_sum example.

parent 913059d2
No related branches found
No related tags found
No related merge requests found
...@@ -40,8 +40,7 @@ Lemma sum_loop_wp `{!heapG Σ} v t l (n : Z) : ...@@ -40,8 +40,7 @@ Lemma sum_loop_wp `{!heapG Σ} v t l (n : Z) :
{{{ RET #(); l #(sum t + n) is_tree v t }}}. {{{ RET #(); l #(sum t + n) is_tree v t }}}.
Proof. Proof.
iIntros (Φ) "[Hl Ht] HΦ". iIntros (Φ) "[Hl Ht] HΦ".
iLöb as "IH" forall (v t l n Φ). wp_rec. wp_let. iInduction t as [n'|tl ? tr] "IH" forall (v l n Φ); wp_rec; wp_let.
destruct t as [n'|tl tr]; simpl in *.
- iDestruct "Ht" as "%"; subst. - iDestruct "Ht" as "%"; subst.
wp_match. wp_load. wp_op. wp_store. wp_match. wp_load. wp_op. wp_store.
by iApply ("HΦ" with "[$Hl]"). by iApply ("HΦ" with "[$Hl]").
...@@ -49,7 +48,7 @@ Proof. ...@@ -49,7 +48,7 @@ Proof.
wp_match. wp_proj. wp_load. wp_match. wp_proj. wp_load.
wp_apply ("IH" with "Hl Htl"). iIntros "[Hl Htl]". wp_apply ("IH" with "Hl Htl"). iIntros "[Hl Htl]".
wp_seq. wp_proj. wp_load. wp_seq. wp_proj. wp_load.
wp_apply ("IH" with "Hl Htr"). iIntros "[Hl Htr]". wp_apply ("IH1" with "Hl Htr"). iIntros "[Hl Htr]".
iApply "HΦ". iSplitL "Hl". iApply "HΦ". iSplitL "Hl".
{ by replace (sum tl + sum tr + n) with (sum tr + (sum tl + n)) by omega. } { by replace (sum tl + sum tr + n) with (sum tr + (sum tl + n)) by omega. }
iExists ll, lr, vl, vr. by iFrame. iExists ll, lr, vl, vr. by iFrame.
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment