diff --git a/CHANGELOG.md b/CHANGELOG.md
index 835085e1cb9171f519531c144752ca385c889f1c..4f286c5b243512867dcdc351a3b15df89876bb2b 100644
--- a/CHANGELOG.md
+++ b/CHANGELOG.md
@@ -64,6 +64,8 @@ HeapLang, which is now in a separate package `coq-iris-heap-lang`.
   inequality instead of RA composition and validity (also in `base_logic` and
   the higher layers).
 * Move `algebra.base` module to `prelude.prelude`.
+* Strengthen `cmra_op_discrete` to assume only `✓{0} (x1 ⋅ x2)` instead of `✓
+  (x1 â‹… x2)`.
 
 **Changes in `bi`:**
 
diff --git a/iris/algebra/cmra.v b/iris/algebra/cmra.v
index cc705a7464b99b5b444d9f7ef15082a84645fd15..d4cb19cce274548aa3e06bbb3955cbc3ea88d338 100644
--- a/iris/algebra/cmra.v
+++ b/iris/algebra/cmra.v
@@ -549,11 +549,11 @@ Qed.
 Lemma cmra_discrete_included_r x y : Discrete y → x ≼{0} y → x ≼ y.
 Proof. intros ? [x' ?]. exists x'. by apply (discrete y). Qed.
 Lemma cmra_op_discrete x1 x2 :
-  ✓ (x1 ⋅ x2) → Discrete x1 → Discrete x2 → Discrete (x1 ⋅ x2).
+  ✓{0} (x1 ⋅ x2) → Discrete x1 → Discrete x2 → Discrete (x1 ⋅ x2).
 Proof.
   intros ??? z Hz.
   destruct (cmra_extend 0 z x1 x2) as (y1&y2&Hz'&?&?); auto; simpl in *.
-  { rewrite -?Hz. by apply cmra_valid_validN. }
+  { rewrite -?Hz. done. }
   by rewrite Hz' (discrete x1 y1) // (discrete x2 y2).
 Qed.