Skip to content

Commit

Permalink
simpl fixes in floyd
Browse files Browse the repository at this point in the history
  • Loading branch information
mansky1 committed Mar 21, 2024
1 parent c2c60e3 commit 5866064
Showing 1 changed file with 4 additions and 2 deletions.
6 changes: 4 additions & 2 deletions floyd/SeparationLogicAsLogic.v
Original file line number Diff line number Diff line change
Expand Up @@ -1413,7 +1413,7 @@ Proof. destruct HI. split3.
(close_precondition (map fst (fn_params f)) (argsassert_of ((Pre_of_funspec (phi i)) x)) ∗ stackframe_of f)
(fn_body f) (frame_ret_assert (function_body_ret_assert (fn_return f) (assert_of ((Post_of_funspec (phi i)) x))) (stackframe_of f)))) as HH.
{ intros. specialize (H1 i); specialize (H2 i). specialize (HE i). subst. unfold semax_body in H.
destruct (phi i); subst. destruct H as [? [? ?]]. split3; auto. }
destruct (phi i); subst. destruct H as [? [? ?]]. split3; simpl; auto. }
clear H H1 H2. destruct HH as [HH1 [HH2 HH3]].
apply (HH3 Hi).
Qed.
Expand Down Expand Up @@ -1499,6 +1499,8 @@ Proof.
apply Clight_assert_lemmas.allp_fun_id_sub; auto.
Qed.

Local Arguments typecheck_expr : simpl never.

Theorem semax_Delta_subsumption {OK_spec: ext_spec OK_ty} {CS: compspecs}:
forall E Delta Delta' P c R,
tycontext_sub Delta Delta' ->
Expand All @@ -1510,7 +1512,7 @@ Proof.
apply andp_ENTAIL; [apply ENTAIL_refl |].
rewrite !bi.later_and; apply andp_ENTAIL, ENTAIL_refl.
unfold local, lift1; normalize.
apply bi.later_mono; eapply Clight_assert_lemmas.tc_expr_sub; eauto.
apply bi.later_mono; eapply Clight_assert_lemmas.tc_expr_sub; auto.
eapply semax_lemmas.typecheck_environ_sub; eauto.
+ eapply AuxDefs.semax_seq; intuition eauto.
+ eapply AuxDefs.semax_break; eauto.
Expand Down

0 comments on commit 5866064

Please sign in to comment.