diff --git a/theories/algebra/frac.v b/theories/algebra/frac.v
index 85543266dc7049a7933bbfac359545b831fe3dfc..4fea0470c2e74174a746630034789f0c15b12890 100644
--- a/theories/algebra/frac.v
+++ b/theories/algebra/frac.v
@@ -55,5 +55,10 @@ Proof. done. Qed.
 Lemma frac_valid' (p : Qp) : ✓ p ↔ (p ≤ 1%Qp)%Qc.
 Proof. done. Qed.
 
-Global Instance is_op_frac q : IsOp' q (q/2)%Qp (q/2)%Qp.
+Global Instance frac_is_op_half q : IsOp' q (q/2)%Qp (q/2)%Qp.
 Proof. by rewrite /IsOp' /IsOp frac_op' Qp_div_2. Qed.
+
+(* This one has a higher precendence than [is_op_op] so we get a [+] instead
+   of an [â‹…]. *)
+Global Instance frac_is_op q1 q2 : IsOp (q1 + q2)%Qp q1 q2.
+Proof. done. Qed.
diff --git a/theories/algebra/numbers.v b/theories/algebra/numbers.v
index b83e36f235fca6a718a5dbede17e0d43340ba827..25893ec9dcfb382a573b67a506a5542d0d09f135 100644
--- a/theories/algebra/numbers.v
+++ b/theories/algebra/numbers.v
@@ -40,7 +40,7 @@ Section nat.
 
   (* This one has a higher precendence than [is_op_op] so we get a [+] instead
      of an [â‹…]. *)
-  Global Instance is_op_plus (n1 n2 : nat) : IsOp (n1 + n2) n1 n2.
+  Global Instance nat_is_op (n1 n2 : nat) : IsOp (n1 + n2) n1 n2.
   Proof. done. Qed.
 End nat.
 
@@ -93,6 +93,10 @@ Section max_nat.
 
   Global Instance : IdemP (=@{max_nat}) (â‹…).
   Proof. intros [x]. rewrite max_nat_op_max. apply f_equal. lia. Qed.
+
+  Global Instance max_nat_is_op (x y : nat) :
+    IsOp (MaxNat (x `max` y)) (MaxNat x) (MaxNat y).
+  Proof. done. Qed.
 End max_nat.
 
 (** ** Natural numbers with [min] as the operation. *)
@@ -145,6 +149,10 @@ Section min_nat.
 
   Global Instance : IdemP (=@{min_nat}) (â‹…).
   Proof. intros [x]. rewrite min_nat_op_min. apply f_equal. lia. Qed.
+
+  Global Instance min_nat_is_op (x y : nat) :
+    IsOp (MinNat (x `min` y)) (MinNat x) (MinNat y).
+  Proof. done. Qed.
 End min_nat.
 
 (** ** Positive integers with [Pos.add] as the operation. *)
@@ -175,4 +183,9 @@ Section positive.
     intros y ??. apply (Pos.add_no_neutral x y). rewrite Pos.add_comm.
     by apply leibniz_equiv.
   Qed.
+
+  (* This one has a higher precendence than [is_op_op] so we get a [+] instead
+     of an [â‹…]. *)
+  Global Instance pos_is_op (x y : positive) : IsOp (x + y)%positive x y.
+  Proof. done. Qed.
 End positive.