diff --git a/theories/proofmode/environments.v b/theories/proofmode/environments.v
index 78a8d28ca7ca2732b8b3712dc85f53573ada2408..4af44c52ae11e399db23c515e6123562733e9f64 100644
--- a/theories/proofmode/environments.v
+++ b/theories/proofmode/environments.v
@@ -263,7 +263,7 @@ Proof. by eexists. Qed.
 Definition envs_entails {PROP : bi} (Δ : envs PROP) (Q : PROP) : Prop :=
   envs_entails_aux.(unseal) PROP (env_intuitionistic Δ) (env_spatial Δ) Q.
 Definition envs_entails_eq :
-  @envs_entails = λ {PROP} (Δ : envs PROP) Q, (of_envs Δ ⊢ Q).
+  @envs_entails = λ PROP (Δ : envs PROP) Q, (of_envs Δ ⊢ Q).
 Proof. by rewrite /envs_entails envs_entails_aux.(seal_eq). Qed.
 Arguments envs_entails {PROP} Δ Q%I : rename.
 Instance: Params (@envs_entails) 1 := {}.