Skip to content
Snippets Groups Projects
invariants.v 6.71 KiB
Newer Older
From stdpp Require Export namespaces.
From iris.proofmode Require Import tactics.
From iris.algebra Require Import gmap.
From iris.base_logic.lib Require Export fancy_updates.
From iris.base_logic.lib Require Import wsat.
Set Default Proof Using "Type".
Import uPred.
Robbert Krebbers's avatar
Robbert Krebbers committed

Ralf Jung's avatar
Ralf Jung committed
(** Semantic Invariants *)
Definition inv_def `{!invG Σ} (N : namespace) (P : iProp Σ) : iProp Σ :=
  (  E, ⌜↑N  E  |={E,E  N}=>  P  ( P ={E  N,E}=∗ True))%I.
Definition inv_aux : seal (@inv_def). by eexists. Qed.
Definition inv {Σ i} := inv_aux.(unseal) Σ i.
Definition inv_eq : @inv = @inv_def := inv_aux.(seal_eq).
Instance: Params (@inv) 3 := {}.
Typeclasses Opaque inv.
Simon Spies's avatar
Simon Spies committed
(** * Invariants *)
Section inv.
  Context `{!invG Σ}.
Ralf Jung's avatar
Ralf Jung committed
  Implicit Types i : positive.
  Implicit Types N : namespace.
  Implicit Types E : coPset.
  Implicit Types P Q R : iProp Σ.
Simon Spies's avatar
Simon Spies committed

Ralf Jung's avatar
Ralf Jung committed
  (** ** Internal model of invariants *)
  Definition own_inv (N : namespace) (P : iProp Σ) : iProp Σ :=
Simon Spies's avatar
Simon Spies committed
    ( i P', i  (N:coPset)    (P'  P)  ownI i P')%I.

Ralf Jung's avatar
Ralf Jung committed
  Lemma own_inv_open E N P :
    N  E  own_inv N P ={E,E∖↑N}=∗  P  ( P ={E∖↑N,E}=∗ True).
Simon Spies's avatar
Simon Spies committed
  Proof.
Ralf Jung's avatar
Ralf Jung committed
    rewrite uPred_fupd_eq /uPred_fupd_def.
Simon Spies's avatar
Simon Spies committed
    iDestruct 1 as (i P') "(Hi & #HP' & #HiP)".
    iDestruct "Hi" as % ?%elem_of_subseteq_singleton.
    rewrite {1 4}(union_difference_L ( N) E) // ownE_op; last set_solver.
    rewrite {1 5}(union_difference_L {[ i ]} ( N)) // ownE_op; last set_solver.
    iIntros "(Hw & [HE $] & $) !> !>".
    iDestruct (ownI_open i with "[$Hw $HE $HiP]") as "($ & HP & HD)".
    iDestruct ("HP'" with "HP") as "$".
    iIntros "HP [Hw $] !> !>". iApply (ownI_close _ P'). iFrame "HD Hw HiP".
    iApply "HP'". iFrame.
  Qed.

Ralf Jung's avatar
Ralf Jung committed
  Lemma fresh_inv_name (E : gset positive) N :  i, i  E  i  (N:coPset).
  Proof.
    exists (coPpick ( N  gset_to_coPset E)).
    rewrite -elem_of_gset_to_coPset (comm and) -elem_of_difference.
    apply coPpick_elem_of=> Hfin.
    eapply nclose_infinite, (difference_finite_inv _ _), Hfin.
    apply gset_to_coPset_finite.
  Qed.

  Lemma own_inv_alloc N E P :  P ={E}=∗ own_inv N P.
Simon Spies's avatar
Simon Spies committed
  Proof.
Ralf Jung's avatar
Ralf Jung committed
    rewrite uPred_fupd_eq. iIntros "HP [Hw $]".
Simon Spies's avatar
Simon Spies committed
    iMod (ownI_alloc (. (N : coPset)) P with "[$HP $Hw]")
      as (i ?) "[$ ?]"; auto using fresh_inv_name.
    do 2 iModIntro. iExists i, P. rewrite -(iff_refl True%I). auto.
  Qed.

Ralf Jung's avatar
Ralf Jung committed
  Lemma own_inv_alloc_open N E P :
    N  E  (|={E, E∖↑N}=> own_inv N P  (P ={E∖↑N, E}=∗ True))%I.
Simon Spies's avatar
Simon Spies committed
  Proof.
Ralf Jung's avatar
Ralf Jung committed
    rewrite uPred_fupd_eq. iIntros (Sub) "[Hw HE]".
Simon Spies's avatar
Simon Spies committed
    iMod (ownI_alloc_open (. (N : coPset)) P with "Hw")
      as (i ?) "(Hw & #Hi & HD)"; auto using fresh_inv_name.
    iAssert (ownE {[i]}  ownE ( N  {[i]})  ownE (E   N))%I
      with "[HE]" as "(HEi & HEN\i & HE\N)".
    { rewrite -?ownE_op; [|set_solver..].
      rewrite assoc_L -!union_difference_L //. set_solver. }
    do 2 iModIntro. iFrame "HE\N". iSplitL "Hw HEi"; first by iApply "Hw".
    iSplitL "Hi".
    { iExists i, P. rewrite -(iff_refl True%I). auto. }
    iIntros "HP [Hw HE\N]".
    iDestruct (ownI_close with "[$Hw $Hi $HP $HD]") as "[$ HEi]".
    do 2 iModIntro. iSplitL; [|done].
    iCombine "HEi HEN\i HE\N" as "HEN".
    rewrite -?ownE_op; [|set_solver..].
    rewrite assoc_L -!union_difference_L //; set_solver.
  Qed.

Ralf Jung's avatar
Ralf Jung committed
  Lemma own_inv_to_inv M P: own_inv M P  -∗ inv M P.
  Proof.
    iIntros "#I". rewrite inv_eq. iIntros (E H).
    iPoseProof (own_inv_open with "I") as "H"; eauto.
  Qed.
Simon Spies's avatar
Simon Spies committed

Ralf Jung's avatar
Ralf Jung committed
  (** ** Public API of invariants *)
  Global Instance inv_contractive N : Contractive (inv N).
Simon Spies's avatar
Simon Spies committed
  Proof. rewrite inv_eq. solve_contractive. Qed.

  Global Instance inv_ne N : NonExpansive (inv N).
  Proof. apply contractive_ne, _. Qed.

Ralf Jung's avatar
Ralf Jung committed
  Global Instance inv_proper N : Proper (equiv ==> equiv) (inv N).
Simon Spies's avatar
Simon Spies committed
  Proof. apply ne_proper, _. Qed.

Ralf Jung's avatar
Ralf Jung committed
  Global Instance inv_persistent N P : Persistent (inv N P).
  Proof. rewrite inv_eq. apply _. Qed.
Simon Spies's avatar
Simon Spies committed

  Lemma inv_acc N P Q:
    inv N P -∗   (P -∗ Q  (Q -∗ P)) -∗ inv N Q.
  Proof.
Ralf Jung's avatar
Ralf Jung committed
    rewrite inv_eq. iIntros "#HI #Acc !>" (E H).
    iMod ("HI" $! E H) as "[HP Hclose]".
    iDestruct ("Acc" with "HP") as "[$ HQP]".
    iIntros "!> HQ". iApply "Hclose". iApply "HQP". done.
Simon Spies's avatar
Simon Spies committed
  Qed.

  Lemma inv_iff N P Q :   (P  Q) -∗ inv N P -∗ inv N Q.
  Proof.
Ralf Jung's avatar
Ralf Jung committed
    iIntros "#HPQ #HI". iApply (inv_acc with "HI").
    iIntros "!> !# HP". iSplitL "HP".
Simon Spies's avatar
Simon Spies committed
    - by iApply "HPQ".
Ralf Jung's avatar
Ralf Jung committed
    - iIntros "HQ". by iApply "HPQ".
Simon Spies's avatar
Simon Spies committed
  Qed.

  Lemma inv_alloc N E P :  P ={E}=∗ inv N P.
  Proof.
Ralf Jung's avatar
Ralf Jung committed
    iIntros "HP". iApply own_inv_to_inv.
    iApply (own_inv_alloc N E with "HP").
Simon Spies's avatar
Simon Spies committed
  Qed.

  Lemma inv_alloc_open N E P :
    N  E  (|={E, E∖↑N}=> inv N P  (P ={E∖↑N, E}=∗ True))%I.
  Proof.
Ralf Jung's avatar
Ralf Jung committed
    iIntros (?). iMod own_inv_alloc_open as "[HI $]"; first done.
    iApply own_inv_to_inv. done.
Simon Spies's avatar
Simon Spies committed
  Qed.

  Lemma inv_open E N P :
    N  E  inv N P ={E,E∖↑N}=∗  P  ( P ={E∖↑N,E}=∗ True).
  Proof.
Ralf Jung's avatar
Ralf Jung committed
    rewrite inv_eq /inv_def; iIntros (?) "#HI". by iApply "HI".
Simon Spies's avatar
Simon Spies committed
  Qed.

Ralf Jung's avatar
Ralf Jung committed
  (** ** Proof mode integration *)
Simon Spies's avatar
Simon Spies committed
  Global Instance into_inv_inv N P : IntoInv (inv N P) N := {}.

  Global Instance into_acc_inv N P E:
    IntoAcc (X := unit) (inv N P)
            (N  E) True (fupd E (E  N)) (fupd (E  N) E)
            (λ _ : (), ( P)%I) (λ _ : (), ( P)%I) (λ _ : (), None).
  Proof.
    rewrite inv_eq /IntoAcc /accessor bi.exist_unit.
    iIntros (?) "#Hinv _". iApply "Hinv"; done.
  Qed.

Ralf Jung's avatar
Ralf Jung committed
  (** ** Derived properties *)
  Lemma inv_open_strong E N P :
    N  E  inv N P ={E,E∖↑N}=∗  P   E',  P ={E',N  E'}=∗ True.
  Proof.
    iIntros (?) "Hinv".
    iPoseProof (inv_open ( N) N P with "Hinv") as "H"; first done.
    rewrite difference_diag_L.
    iPoseProof (fupd_mask_frame_r _ _ (E   N) with "H") as "H"; first set_solver.
    rewrite left_id_L -union_difference_L //. iMod "H" as "[$ H]"; iModIntro.
    iIntros (E') "HP".
    iPoseProof (fupd_mask_frame_r _ _ E' with "(H HP)") as "H"; first set_solver.
    by rewrite left_id_L.
  Qed.

Simon Spies's avatar
Simon Spies committed
  Lemma inv_open_timeless E N P `{!Timeless P} :
    N  E  inv N P ={E,E∖↑N}=∗ P  (P ={E∖↑N,E}=∗ True).
  Proof.
    iIntros (?) "Hinv". iMod (inv_open with "Hinv") as "[>HP Hclose]"; auto.
    iIntros "!> {$HP} HP". iApply "Hclose"; auto.
  Qed.

Ralf Jung's avatar
Ralf Jung committed
  Lemma inv_sep_l N P Q : inv N (P  Q) -∗ inv N P.
Simon Spies's avatar
Simon Spies committed
  Proof.
Ralf Jung's avatar
Ralf Jung committed
    iIntros "#HI". iApply inv_acc; eauto.
    iIntros "!> !# [$ $] $".
Simon Spies's avatar
Simon Spies committed
  Qed.

Ralf Jung's avatar
Ralf Jung committed
  Lemma inv_sep_r N P Q : inv N (P  Q) -∗ inv N Q.
Simon Spies's avatar
Simon Spies committed
  Proof.
Ralf Jung's avatar
Ralf Jung committed
    rewrite (comm _ P Q). eapply inv_sep_l.
Simon Spies's avatar
Simon Spies committed
  Qed.

Ralf Jung's avatar
Ralf Jung committed
  Lemma inv_sep N P Q : inv N (P  Q) -∗ inv N P  inv N Q.
Simon Spies's avatar
Simon Spies committed
  Proof.
    iIntros "#H".
Ralf Jung's avatar
Ralf Jung committed
    iPoseProof (inv_sep_l with "H") as "$".
    iPoseProof (inv_sep_r with "H") as "$".
Simon Spies's avatar
Simon Spies committed
  Qed.
End inv.