diff --git a/_CoqProject b/_CoqProject
index e587aa9aaa5622b2a0ef7d38a31d2f61e8139e40..b397e30d55f3115ec244e87e4a51c6f3861e662c 100644
--- a/_CoqProject
+++ b/_CoqProject
@@ -51,7 +51,6 @@ theories/base_logic/bi.v
 theories/base_logic/derived.v
 theories/base_logic/proofmode.v
 theories/base_logic/base_logic.v
-theories/base_logic/double_negation.v
 theories/base_logic/lib/iprop.v
 theories/base_logic/lib/own.v
 theories/base_logic/lib/saved_prop.v
diff --git a/theories/base_logic/bi.v b/theories/base_logic/bi.v
index 3b8c338ec851cc30dd6b33144f5cf447e9934df0..16d5b2cf2f8760ace873acef32cc3803e599629e 100644
--- a/theories/base_logic/bi.v
+++ b/theories/base_logic/bi.v
@@ -128,20 +128,6 @@ Qed.
 Global Instance uPred_plainlyC M : BiPlainly (uPredSI M) :=
   {| bi_plainly_mixin := uPred_plainly_mixin M |}.
 
-Lemma uPred_bupd_mixin M : BiBUpdMixin (uPredI M) uPred_bupd.
-Proof.
-  split.
-  - exact: bupd_ne.
-  - exact: bupd_intro.
-  - exact: bupd_mono.
-  - exact: bupd_trans.
-  - exact: bupd_frame_r.
-Qed.
-Global Instance uPred_bi_bupd M : BiBUpd (uPredI M) := {| bi_bupd_mixin := uPred_bupd_mixin M |}.
-
-Global Instance uPred_bi_bupd_plainly M : BiBUpdPlainly (uPredSI M).
-Proof. exact: bupd_plainly. Qed.
-
 (** extra BI instances *)
 
 Global Instance uPred_affine M : BiAffine (uPredI M) | 0.
@@ -181,9 +167,10 @@ Lemma ownM_unit P : P ⊢ (uPred_ownM ε).
 Proof. exact: uPred_primitive.ownM_unit. Qed.
 Lemma later_ownM a : ▷ uPred_ownM a ⊢ ∃ b, uPred_ownM b ∧ ▷ (a ≡ b).
 Proof. exact: uPred_primitive.later_ownM. Qed.
-Lemma bupd_ownM_updateP x (Φ : M → Prop) :
-  x ~~>: Φ → uPred_ownM x ⊢ |==> ∃ y, ⌜Φ y⌝ ∧ uPred_ownM y.
-Proof. exact: uPred_primitive.bupd_ownM_updateP. Qed.
+Lemma ownM_updateP x (Φ : M → Prop) R :
+  x ~~>: Φ →
+  uPred_ownM x ∗ (∀ y, ⌜Φ y⌝ -∗ uPred_ownM y -∗ ■ R) ⊢ ■ R.
+Proof. exact: uPred_primitive.ownM_updateP. Qed.
 
 Lemma ownM_valid (a : M) : uPred_ownM a ⊢ ✓ a.
 Proof. exact: uPred_primitive.ownM_valid. Qed.
diff --git a/theories/base_logic/derived.v b/theories/base_logic/derived.v
index d3ff12d81d6622b48e7e5a107fbfd1e62512dab8..28f976bb7e18b41613cca28b261b05fd67ec3ef0 100644
--- a/theories/base_logic/derived.v
+++ b/theories/base_logic/derived.v
@@ -5,6 +5,31 @@ Import bi base_logic.bi.uPred.
 
 (** Derived laws for Iris-specific primitive connectives (own, valid).
     This file does NOT unseal! *)
+Definition uPred_bupd {M} (P : uPred M) : uPred M :=
+  (∀ Q, (P -∗ ■ Q) -∗ ■ Q)%I.
+Lemma uPred_bupd_mixin M : BiBUpdMixin (uPredI M) uPred_bupd.
+Proof.
+  split; rewrite /bupd /uPred_bupd.
+  - solve_proper.
+  - intros P. apply bi.forall_intro=> Q. apply bi.wand_intro_l.
+    by rewrite bi.wand_elim_l.
+  - intros P Q H. apply bi.forall_mono=> R. by repeat f_equiv.
+  - intros P. apply bi.forall_intro=> Q. apply bi.wand_intro_l.
+    rewrite !(bi.forall_elim Q). etrans; [apply bi.sep_mono_l|apply bi.wand_elim_r].
+    apply bi.wand_intro_r. by rewrite bi.wand_elim_r.
+  - intros P R. apply bi.forall_intro=> Q. apply bi.wand_intro_l.
+    rewrite (bi.forall_elim Q). rewrite !(comm _ _ R) assoc.
+    by rewrite -bi.wand_curry bi.wand_elim_l bi.wand_elim_r.
+Qed.
+Global Instance uPred_bi_bupd M : BiBUpd (uPredI M) :=
+  {| bi_bupd_mixin := uPred_bupd_mixin M |}.
+
+Global Instance uPred_bi_bupd_plainly M : BiBUpdPlainly (uPredSI M).
+Proof.
+  intros P. rewrite /bupd /bi_bupd_bupd /= /uPred_bupd.
+  rewrite (bi.forall_elim P) -(bi.entails_wand' (â–  P)%I (â–  P)%I) // bi.emp_wand.
+  apply (plainly_elim _).
+Qed.
 
 Module uPred.
 Section derived.
@@ -53,6 +78,15 @@ Proof.
     first by rewrite persistently_elim.
   apply:persistently_cmra_valid_1.
 Qed.
+
+Lemma bupd_ownM_updateP x (Φ : M → Prop) :
+  x ~~>: Φ → uPred_ownM x ⊢ |==> ∃ y, ⌜Φ y⌝ ∧ uPred_ownM y.
+Proof.
+  intros Hup. apply bi.forall_intro=> R. apply bi.wand_intro_r.
+  etrans; [apply bi.sep_mono_r|by eapply ownM_updateP].
+  apply bi.forall_intro=> y. rewrite -(bi.exist_intro y).
+  by rewrite bi.persistent_and_sep bi.wand_curry.
+Qed.
 Lemma bupd_ownM_update x y : x ~~> y → uPred_ownM x ⊢ |==> uPred_ownM y.
 Proof.
   intros; rewrite (bupd_ownM_updateP _ (y =)); last by apply cmra_update_updateP.
diff --git a/theories/base_logic/double_negation.v b/theories/base_logic/double_negation.v
deleted file mode 100644
index 4ebe5cccc7ae03383bc76cf0c0be2760fb0165c9..0000000000000000000000000000000000000000
--- a/theories/base_logic/double_negation.v
+++ /dev/null
@@ -1,370 +0,0 @@
-From iris.base_logic Require Import base_logic.
-Set Default Proof Using "Type".
-
-(* In this file we show that the bupd can be thought of a kind of
-   step-indexed double-negation when our meta-logic is classical *)
-Definition uPred_nnupd {M} (P: uPred M) : uPred M :=
-  ∀ n, (P -∗ ▷^n False) -∗ ▷^n False.
-
-Notation "|=n=> Q" := (uPred_nnupd Q)
-  (at level 99, Q at level 200, format "|=n=>  Q") : bi_scope.
-Notation "P =n=> Q" := (P ⊢ |=n=> Q)
-  (at level 99, Q at level 200, only parsing) : stdpp_scope.
-Notation "P =n=∗ Q" := (P -∗ |=n=> Q)%I
-  (at level 99, Q at level 200, format "P  =n=∗  Q") : bi_scope.
-
-(* Our goal is to prove that:
-  (1) |=n=> has (nearly) all the properties of the |==> modality that are used in Iris
-  (2) If our meta-logic is classical, then |=n=> and |==> are equivalent
-*)
-
-Section bupd_nnupd.
-Context {M : ucmraT}.
-Implicit Types φ : Prop.
-Implicit Types P Q : uPred M.
-Implicit Types A : Type.
-Implicit Types x : M.
-Import uPred.
-
-(* Helper lemmas about iterated later modalities *)
-Lemma laterN_big n a x φ: ✓{n} x →  a ≤ n → (▷^a ⌜φ⌝ : uPred M)%I n x → φ.
-Proof.
-  induction 2 as [| ?? IHle].
-  - induction a; repeat (rewrite //= || uPred.unseal).
-    intros Hlater. apply IHa; auto using cmra_validN_S.
-    move:Hlater; repeat (rewrite //= || uPred.unseal).
-  - intros. apply IHle; auto using cmra_validN_S.
-    eapply uPred_mono; eauto using cmra_validN_S.
-Qed.
-
-Lemma laterN_small n a x φ: ✓{n} x →  n < a → (▷^a ⌜φ⌝ : uPred M)%I n x.
-Proof.
-  induction 2.
-  - induction n as [| n IHn]; [| move: IHn];
-      repeat (rewrite //= || uPred.unseal).
-    naive_solver eauto using cmra_validN_S.
-  - induction n as [| n IHn]; [| move: IHle];
-      repeat (rewrite //= || uPred.unseal).
-    red; rewrite //=. intros.
-    eapply (uPred_mono _ _ (S n)); eauto using cmra_validN_S.
-Qed.
-
-(* It is easy to show that most of the basic properties of bupd that
-   are used throughout Iris hold for nnupd.
-
-   In fact, the first three properties that follow hold for any
-   modality of the form (- -∗ Q) -∗ Q for arbitrary Q. The situation
-   here is slightly different, because nnupd is of the form
-   ∀ n, (- -∗ (Q n)) -∗ (Q n), but the proofs carry over straightforwardly.
-
- *)
-
-Lemma nnupd_intro P : P =n=> P.
-Proof. apply forall_intro=>?. apply wand_intro_l, wand_elim_l. Qed.
-Lemma nnupd_mono P Q : (P ⊢ Q) → (|=n=> P) =n=> Q.
-Proof.
-  intros HPQ. apply forall_intro=>n.
-  apply wand_intro_l.  rewrite -{1}HPQ.
-  rewrite /uPred_nnupd (forall_elim n).
-  apply wand_elim_r.
-Qed.
-Lemma nnupd_frame_r P R : (|=n=> P) ∗ R =n=> P ∗ R.
-Proof.
-  apply forall_intro=>n. apply wand_intro_r.
-  rewrite (comm _ P) -wand_curry.
-  rewrite /uPred_nnupd (forall_elim n).
-  by rewrite -assoc wand_elim_r wand_elim_l.
-Qed.
-Lemma nnupd_ownM_updateP x (Φ : M → Prop) :
-  x ~~>: Φ → uPred_ownM x =n=> ∃ y, ⌜Φ y⌝ ∧ uPred_ownM y.
-Proof.
-  intros Hbupd. split. rewrite /uPred_nnupd. repeat uPred.unseal.
-  intros n y ? Hown a.
-  red; rewrite //= => n' yf ??.
-  inversion Hown as (x'&Hequiv).
-  edestruct (Hbupd n' (Some (x' â‹… yf))) as (y'&?&?); eauto.
-  { by rewrite //= assoc -(dist_le _ _ _ _ Hequiv). }
-  case (decide (a ≤ n')).
-  - intros Hle Hwand.
-    exfalso. eapply laterN_big; last (uPred.unseal; eapply (Hwand n' (y' â‹… x'))); eauto.
-    * rewrite comm -assoc. done.
-    * rewrite comm -assoc. done.
-    * exists y'. split=>//. by exists x'.
- - intros; assert (n' < a). lia.
-    move: laterN_small. uPred.unseal.
-    naive_solver.
-Qed.
-
-(* However, the transitivity property seems to be much harder to
-   prove. This is surprising, because transitivity does hold for
-   modalities of the form (- -∗ Q) -∗ Q. What goes wrong when we quantify
-   now over n?
- *)
-
-Remark nnupd_trans P: (|=n=> |=n=> P) ⊢ (|=n=> P).
-Proof.
-  rewrite /uPred_nnupd.
-  apply forall_intro=>a. apply wand_intro_l.
-  rewrite (forall_elim a).
-  rewrite (nnupd_intro (P -∗ _)).
-  rewrite /uPred_nnupd.
-  (* Oops -- the exponents of the later modality don't match up! *)
-Abort.
-
-(* Instead, we will need to prove this in the model. We start by showing that
-   nnupd is the limit of a the following sequence:
-
-   (- -∗ False) - ∗ False,
-   (- -∗ ▷ False) - ∗ ▷ False ∧ (- -∗ False) - ∗ False,
-   (- -∗ ▷^2 False) - ∗ ▷^2 False ∧ (- -∗ ▷ False) - ∗ ▷ False ∧ (- -∗ False) - ∗ False,
-   ...
-
-   Then, it is easy enough to show that each of the uPreds in this sequence
-   is transitive. It turns out that this implies that nnupd is transitive. *)
-
-
-(* The definition of the sequence above: *)
-Fixpoint uPred_nnupd_k {M} k (P: uPred M) : uPred M :=
-  ((P -∗ ▷^k False) -∗ ▷^k False) ∧
-  match k with
-    O => True
-  | S k' => uPred_nnupd_k k' P
-  end.
-
-Notation "|=n=>_ k Q" := (uPred_nnupd_k k Q)
-  (at level 99, k at level 9, Q at level 200, format "|=n=>_ k  Q") : bi_scope.
-
-
-(* One direction of the limiting process is easy -- nnupd implies nnupd_k for each k *)
-Lemma nnupd_trunc1 k P: (|=n=> P) ⊢ |=n=>_k P.
-Proof.
-  induction k.
-  - rewrite /uPred_nnupd_k /uPred_nnupd.
-    rewrite (forall_elim 0) //= right_id //.
-  - simpl. apply and_intro; auto.
-    rewrite /uPred_nnupd.
-    rewrite (forall_elim (S k)) //=.
-Qed.
-
-Lemma nnupd_k_elim n k P: n ≤ k → ((|=n=>_k P) ∗ (P -∗ (▷^n False)) ⊢  (▷^n False))%I.
-Proof.
-  induction k.
-  - inversion 1; subst; rewrite //= ?right_id. apply wand_elim_l.
-  - inversion 1; subst; rewrite //= ?right_id.
-    * rewrite and_elim_l. apply wand_elim_l.
-    * rewrite and_elim_r IHk //.
-Qed.
-
-Lemma nnupd_k_unfold k P:
-  (|=n=>_(S k) P) ⊣⊢ ((P -∗ (▷^(S k) False)) -∗ (▷^(S k) False)) ∧ (|=n=>_k P).
-Proof. done.  Qed.
-Lemma nnupd_k_unfold' k P n x:
-  (|=n=>_(S k) P)%I n x ↔ (((P -∗ (▷^(S k) False)) -∗ (▷^(S k) False)) ∧ (|=n=>_k P))%I n x.
-Proof. done.  Qed.
-
-Lemma nnupd_k_weaken k P: (|=n=>_(S k) P) ⊢ |=n=>_k P.
-Proof. by rewrite nnupd_k_unfold and_elim_r. Qed.
-
-(* Now we are ready to show nnupd is the limit -- ie, for each k, it is within distance k
-   of the kth term of the sequence *)
-Lemma nnupd_nnupd_k_dist k P: (|=n=> P)%I ≡{k}≡ (|=n=>_k P)%I.
-  split; intros n' x Hle Hx. split.
-  - by apply (nnupd_trunc1 k).
-  - revert n' x Hle Hx; induction k; intros n' x Hle Hx;
-      rewrite ?nnupd_k_unfold' /uPred_nnupd.
-    * rewrite //=. unseal.
-      inversion Hle; subst.
-      intros (HnnP&_) n k' x' ?? HPF.
-      case (decide (k' < n)).
-      ** move: laterN_small; uPred.unseal; naive_solver.
-      ** intros. exfalso. eapply HnnP; eauto.
-         assert (n ≤ k'). lia.
-         intros n'' x'' ???.
-         specialize (HPF n'' x''). exfalso.
-         eapply laterN_big; last (unseal; eauto).
-         eauto. lia.
-    * inversion Hle; simpl; subst.
-      ** unseal. intros (HnnP&HnnP_IH) n k' x' ?? HPF.
-         case (decide (k' < n)).
-         *** move: laterN_small; uPred.unseal; naive_solver.
-         *** intros. exfalso. assert (n ≤ k'). lia.
-             assert (n = S k ∨ n < S k) as [->|] by lia.
-             **** eapply laterN_big; eauto; unseal.
-                  eapply HnnP; eauto. move: HPF; by unseal.
-             **** move:nnupd_k_elim. unseal. intros Hnnupdk.
-                  eapply laterN_big; eauto. unseal.
-                  eapply (Hnnupdk n k); first lia; eauto.
-                  exists x, x'. split_and!; eauto. eapply uPred_mono; eauto.
-      ** intros HP. eapply IHk; auto.
-         move:HP. unseal. intros (?&?); naive_solver.
-Qed.
-
-(* nnupd_k has a number of structural properties, including transitivity *)
-Lemma nnupd_k_intro k P: P ⊢ (|=n=>_k P).
-Proof.
-  induction k; rewrite //= ?right_id.
-  - apply wand_intro_l. apply wand_elim_l.
-  - apply and_intro; auto.
-    apply wand_intro_l. apply wand_elim_l.
-Qed.
-
-Lemma nnupd_k_mono k P Q: (P ⊢ Q) → (|=n=>_k P) ⊢ (|=n=>_k Q).
-Proof.
-  induction k; rewrite //= ?right_id=>HPQ.
-  - do 2 (apply wand_mono; auto).
-  - apply and_mono; auto; do 2 (apply wand_mono; auto).
-Qed.
-Instance nnupd_k_mono' k: Proper ((⊢) ==> (⊢)) (@uPred_nnupd_k M k).
-Proof. by intros P P' HP; apply nnupd_k_mono. Qed.
-
-Instance nnupd_k_ne k : NonExpansive (@uPred_nnupd_k M k).
-Proof. intros n. induction k; rewrite //= ?right_id=>P P' HP; by rewrite HP. Qed.
-Lemma nnupd_k_proper k P Q: (P ⊣⊢ Q) → (|=n=>_k P) ⊣⊢ (|=n=>_k Q).
-Proof. intros HP; apply (anti_symm (⊢)); eapply nnupd_k_mono; by rewrite HP. Qed.
-Instance nnupd_k_proper' k: Proper ((⊣⊢) ==> (⊣⊢)) (@uPred_nnupd_k M k).
-Proof. by intros P P' HP; apply nnupd_k_proper. Qed.
-
-Lemma nnupd_k_trans k P: (|=n=>_k |=n=>_k P) ⊢ (|=n=>_k P).
-Proof.
-  revert P.
-  induction k; intros P.
-  - rewrite //= ?right_id. apply wand_intro_l.
-    rewrite {1}(nnupd_k_intro 0 (P -∗ False)%I) //= ?right_id. apply wand_elim_r.
-  - rewrite {2}(nnupd_k_unfold k P).
-    apply and_intro.
-    * rewrite (nnupd_k_unfold k P). rewrite and_elim_l.
-      rewrite nnupd_k_unfold. rewrite and_elim_l.
-      apply wand_intro_l.
-      rewrite {1}(nnupd_k_intro (S k) (P -∗ ▷^(S k) (False)%I)).
-      rewrite nnupd_k_unfold and_elim_l. apply wand_elim_r.
-    * do 2 rewrite nnupd_k_weaken //.
-Qed.
-
-Lemma nnupd_trans P : (|=n=> |=n=> P) =n=> P.
-Proof.
-  split=> n x ? Hnn.
-  eapply nnupd_nnupd_k_dist in Hnn; eauto.
-  eapply (nnupd_k_ne (n) n ((|=n=>_(n) P)%I)) in Hnn; eauto;
-    [| symmetry; eapply nnupd_nnupd_k_dist].
-  eapply nnupd_nnupd_k_dist; eauto.
-  by apply nnupd_k_trans.
-Qed.
-
-(* Now that we have shown nnupd has all of the desired properties of
-   bupd, we go further and show it is in fact equivalent to bupd! The
-   direction from bupd to nnupd is similar to the proof of
-   nnupd_ownM_updateP *)
-
-Lemma bupd_nnupd P: (|==> P) ⊢ |=n=> P.
-Proof.
-  split. rewrite /uPred_nnupd. repeat uPred.unseal. intros n x ? Hbupd a.
-  red; rewrite //= => n' yf ??.
-  edestruct Hbupd as (x'&?&?); eauto.
-  case (decide (a ≤ n')).
-  - intros Hle Hwand.
-    exfalso. eapply laterN_big; last (uPred.unseal; eapply (Hwand n' x')); eauto.
-    * rewrite comm. done.
-    * rewrite comm. done.
-  - intros; assert (n' < a). lia.
-    move: laterN_small. uPred.unseal.
-    naive_solver.
-Qed.
-
-(* However, the other direction seems to need a classical axiom: *)
-Section classical.
-Context (not_all_not_ex: ∀ (P : M → Prop), ¬ (∀ n : M, ¬ P n) → ∃ n : M, P n).
-Lemma nnupd_bupd P:  (|=n=> P) ⊢ (|==> P).
-Proof using Type*.
-  rewrite /uPred_nnupd.
-  split. uPred.unseal; red; rewrite //=.
-  intros n x ? Hforall k yf Hle ?.
-  apply not_all_not_ex.
-  intros Hfal.
-  specialize (Hforall k k).
-  eapply laterN_big; last (uPred.unseal; red; rewrite //=; eapply Hforall);
-    eauto.
-  red; rewrite //= => n' x' ???.
-  case (decide (n' = k)); intros.
-  - subst. exfalso. eapply Hfal. rewrite (comm op); eauto.
-  - assert (n' < k). lia.
-    move: laterN_small. uPred.unseal. naive_solver.
-Qed.
-End classical.
-
-(* We might wonder whether we can prove an adequacy lemma for nnupd. We could combine
-   the adequacy lemma for bupd with the previous result to get adquacy for nnupd, but
-   this would rely on the classical axiom we needed to prove the equivalence! Can
-   we establish adequacy without axioms? Unfortunately not, because adequacy for
-   nnupd would imply double negation elimination, which is classical: *)
-
-Lemma nnupd_dne φ: (|=n=> ⌜¬¬ φ → φ⌝: uPred M)%I.
-Proof.
-  rewrite /uPred_nnupd. apply forall_intro=>n.
-  apply wand_intro_l. rewrite ?right_id.
-  assert (∀ φ, ¬¬¬¬φ → ¬¬φ) by naive_solver.
-  assert (Hdne: ¬¬ (¬¬φ → φ)) by naive_solver.
-  split. unseal. intros n' ?? Hupd.
-  case (decide (n' < n)).
-  - intros. move: laterN_small. unseal. naive_solver.
-  - intros. assert (n ≤ n'). lia.
-    exfalso. specialize (Hupd n' ε).
-    eapply Hdne. intros Hfal.
-    eapply laterN_big; eauto.
-    unseal. rewrite right_id in Hupd *; naive_solver.
-Qed.
-
-(* Nevertheless, we can prove a weaker form of adequacy (which is equvialent to adequacy
-   under classical axioms) directly without passing through the proofs for bupd: *)
-Lemma adequacy_helper1 P n k x:
-  ✓{S n + k} x → ¬¬ (Nat.iter (S n) (λ P, |=n=> ▷ P)%I P (S n + k) x)
-            → ¬¬ (∃ x', ✓{n + k} (x') ∧ Nat.iter n (λ P, |=n=> ▷ P)%I P (n + k) (x')).
-Proof.
-  revert k P x. induction n.
-  - rewrite /uPred_nnupd. unseal=> k P x Hx Hf1 Hf2.
-    eapply Hf1. intros Hf3.
-    eapply (laterN_big (S k) (S k)); eauto.
-    specialize (Hf3 (S k) (S k) ε). rewrite right_id in Hf3 *. unseal.
-    intros Hf3. eapply Hf3; eauto.
-    intros ??? Hx'. rewrite left_id in Hx' *=> Hx'.
-    assert (n' < S k ∨ n' = S k) as [|] by lia.
-    * intros. move:(laterN_small n' (S k) x' False). rewrite //=. unseal. intros Hsmall.
-      eapply Hsmall; eauto.
-    * subst. intros. exfalso. eapply Hf2. exists x'. split; eauto using cmra_validN_S.
-  - intros k P x Hx. rewrite ?Nat_iter_S_r.
-    replace (S (S n) + k) with (S n + (S k)) by lia.
-    replace (S n + k) with (n + (S k)) by lia.
-    intros. eapply IHn. replace (S n + S k) with (S (S n) + k) by lia. eauto.
-    rewrite ?Nat_iter_S_r. eauto.
-Qed.
-
-Lemma adequacy_helper2 P n k x:
-  ✓{S n + k} x → ¬¬ (Nat.iter (S n) (λ P, |=n=> ▷ P)%I P (S n + k) x)
-            → ¬¬ (∃ x', ✓{k} (x') ∧ Nat.iter 0 (λ P, |=n=> ▷ P)%I P k (x')).
-Proof.
-  revert x. induction n.
-  - specialize (adequacy_helper1 P 0). rewrite //=. naive_solver.
-  - intros ?? Hfal%adequacy_helper1; eauto using cmra_validN_S.
-    intros Hfal'. eapply Hfal. intros (x''&?&?).
-    eapply IHn; eauto.
-Qed.
-
-Lemma adequacy φ n : Nat.iter n (λ P, |=n=> ▷ P)%I ⌜φ⌝%I → ¬¬ φ.
-Proof.
-  cut (∀ x, ✓{S n} x → Nat.iter n (λ P, |=n=> ▷ P)%I ⌜φ⌝%I (S n) x → ¬¬φ).
-  { intros help H. eapply (help ∅); eauto using ucmra_unit_validN.
-    eapply H; eauto using ucmra_unit_validN. by unseal. }
-  destruct n.
-  - rewrite //=; unseal; auto.
-  - intros ??? Hfal.
-    eapply (adequacy_helper2 _ n 1); (replace (S n + 1) with (S (S n)) by lia); eauto.
-    unseal. intros (x'&?&Hphi). simpl in *.
-    eapply Hfal. auto.
-Qed.
-
-(* Open question:
-
-   Do the basic properties of the |==> modality (bupd_intro, bupd_mono, rvs_trans, rvs_frame_r,
-      bupd_ownM_updateP, and adequacy) uniquely characterize |==>?
-*)
-
-End bupd_nnupd.
diff --git a/theories/base_logic/upred.v b/theories/base_logic/upred.v
index 6f04ccb5499337ada42a3eedcda6efbf1ac84db2..5e12486cd2de8399c14d1caa0bc6bc5dd4e87e3d 100644
--- a/theories/base_logic/upred.v
+++ b/theories/base_logic/upred.v
@@ -322,21 +322,6 @@ Definition uPred_cmra_valid {M A} := uPred_cmra_valid_aux.(unseal) M A.
 Definition uPred_cmra_valid_eq :
   @uPred_cmra_valid = @uPred_cmra_valid_def := uPred_cmra_valid_aux.(seal_eq).
 
-Program Definition uPred_bupd_def {M} (Q : uPred M) : uPred M :=
-  {| uPred_holds n x := ∀ k yf,
-      k ≤ n → ✓{k} (x ⋅ yf) → ∃ x', ✓{k} (x' ⋅ yf) ∧ Q k x' |}.
-Next Obligation.
-  intros M Q n1 n2 x1 x2 HQ [x3 Hx] Hn k yf Hk.
-  rewrite (dist_le _ _ _ _ Hx); last lia. intros Hxy.
-  destruct (HQ k (x3 â‹… yf)) as (x'&?&?); [auto|by rewrite assoc|].
-  exists (x' â‹… x3); split; first by rewrite -assoc.
-  eauto using uPred_mono, cmra_includedN_l.
-Qed.
-Definition uPred_bupd_aux : seal (@uPred_bupd_def). by eexists. Qed.
-Definition uPred_bupd {M} := uPred_bupd_aux.(unseal) M.
-Definition uPred_bupd_eq :
-  @uPred_bupd = @uPred_bupd_def := uPred_bupd_aux.(seal_eq).
-
 (** Global uPred-specific Notation *)
 Notation "✓ x" := (uPred_cmra_valid x) (at level 20) : bi_scope.
 
@@ -348,7 +333,7 @@ Definition unseal_eqs :=
   (uPred_pure_eq, uPred_and_eq, uPred_or_eq, uPred_impl_eq, uPred_forall_eq,
   uPred_exist_eq, uPred_internal_eq_eq, uPred_sep_eq, uPred_wand_eq,
   uPred_plainly_eq, uPred_persistently_eq, uPred_later_eq, uPred_ownM_eq,
-  uPred_cmra_valid_eq, @uPred_bupd_eq).
+  uPred_cmra_valid_eq).
 Ltac unseal :=
   rewrite !unseal_eqs /=.
 
@@ -381,7 +366,6 @@ Notation "â–¡ P" := (uPred_persistently P) : bi_scope.
 Notation "â–  P" := (uPred_plainly P) : bi_scope.
 Notation "x ≡ y" := (uPred_internal_eq x y) : bi_scope.
 Notation "â–· P" := (uPred_later P) : bi_scope.
-Notation "|==> P" := (uPred_bupd P) : bi_scope.
 
 (** Entailment *)
 Lemma entails_po : PreOrder (⊢).
@@ -495,14 +479,6 @@ Proof.
   by rewrite (dist_le _ _ _ _ Ha); last lia.
 Qed.
 
-Lemma bupd_ne : NonExpansive (@uPred_bupd M).
-Proof.
-  intros n P Q HPQ.
-  unseal; split=> n' x; split; intros HP k yf ??;
-    destruct (HP k yf) as (x'&?&?); auto;
-    exists x'; split; auto; apply HPQ; eauto using cmra_validN_op_l.
-Qed.
-
 (** Introduction and elimination rules *)
 Lemma pure_intro φ P : φ → P ⊢ ⌜φ⌝.
 Proof. by intros ?; unseal; split. Qed.
@@ -710,35 +686,6 @@ Proof.
   unseal=> ?. split=> n x ?. by apply (discrete_iff n).
 Qed.
 
-(** Basic update modality *)
-Lemma bupd_intro P : P ⊢ |==> P.
-Proof.
-  unseal. split=> n x ? HP k yf ?; exists x; split; first done.
-  apply uPred_mono with n x; eauto using cmra_validN_op_l.
-Qed.
-Lemma bupd_mono P Q : (P ⊢ Q) → (|==> P) ⊢ |==> Q.
-Proof.
-  unseal. intros HPQ; split=> n x ? HP k yf ??.
-  destruct (HP k yf) as (x'&?&?); eauto.
-  exists x'; split; eauto using uPred_in_entails, cmra_validN_op_l.
-Qed.
-Lemma bupd_trans P : (|==> |==> P) ⊢ |==> P.
-Proof. unseal; split; naive_solver. Qed.
-Lemma bupd_frame_r P R : (|==> P) ∗ R ⊢ |==> P ∗ R.
-Proof.
-  unseal; split; intros n x ? (x1&x2&Hx&HP&?) k yf ??.
-  destruct (HP k (x2 â‹… yf)) as (x'&?&?); eauto.
-  { by rewrite assoc -(dist_le _ _ _ _ Hx); last lia. }
-  exists (x' â‹… x2); split; first by rewrite -assoc.
-  exists x', x2. eauto using uPred_mono, cmra_validN_op_l, cmra_validN_op_r.
-Qed.
-Lemma bupd_plainly P : (|==> ■ P) ⊢ P.
-Proof.
-  unseal; split => n x Hnx /= Hng.
-  destruct (Hng n ε) as [? [_ Hng']]; try rewrite right_id; auto.
-  eapply uPred_mono; eauto using ucmra_unit_leastN.
-Qed.
-
 (** Own *)
 Lemma ownM_op (a1 a2 : M) :
   uPred_ownM (a1 ⋅ a2) ⊣⊢ uPred_ownM a1 ∗ uPred_ownM a2.
@@ -764,14 +711,16 @@ Proof.
   exists a'. rewrite Hx. eauto using cmra_includedN_l.
 Qed.
 
-Lemma bupd_ownM_updateP x (Φ : M → Prop) :
-  x ~~>: Φ → uPred_ownM x ⊢ |==> ∃ y, ⌜Φ y⌝ ∧ uPred_ownM y.
+Lemma ownM_updateP x (Φ : M → Prop) R :
+  x ~~>: Φ →
+  uPred_ownM x ∗ (∀ y, ⌜Φ y⌝ -∗ uPred_ownM y -∗ ■ R) ⊢ ■ R.
 Proof.
-  unseal=> Hup; split=> n x2 ? [x3 Hx] k yf ??.
-  destruct (Hup k (Some (x3 â‹… yf))) as (y&?&?); simpl in *.
-  { rewrite /= assoc -(dist_le _ _ _ _ Hx); auto. }
-  exists (y â‹… x3); split; first by rewrite -assoc.
-  exists y; eauto using cmra_includedN_l.
+  unseal=> Hup; split; intros n z Hv (?&z2&?&[z1 ?]&HR); ofe_subst.
+  destruct (Hup n (Some (z1 â‹… z2))) as (y&?&?); simpl in *.
+  { by rewrite assoc. }
+  refine (HR y n z1 _ _ _ n y _ _ _); auto.
+  - rewrite comm. by eapply cmra_validN_op_r.
+  - by rewrite (comm _ _ y) (comm _ z2).
 Qed.
 
 (** Valid *)