@@ -292,9 +292,9 @@ recommended_spelling "PProd" for "×'" in [PProd, «term_×'_»]
292292@[inherit_doc] infixl :75 " >>> " => HShiftRight.hShiftRight
293293@[inherit_doc] infixr :80 " ^ " => HPow.hPow
294294@[inherit_doc] infixl :65 " ++ " => HAppend.hAppend
295- @[inherit_doc] prefix :75 "-" => Neg.neg
295+ @[inherit_doc] prefix :75 "-" => Neg.neg
296296@[inherit_doc] prefix :100 "~~~" => Complement.complement
297- @[inherit_doc] postfix :max "⁻¹" => Inv.inv
297+ @[inherit_doc] postfix :max "⁻¹" => Inv.inv
298298
299299/-!
300300 Remark: the infix commands above ensure a delaborator is generated for each relations.
@@ -312,7 +312,6 @@ macro_rules | `($x % $y) => `(binop% HMod.hMod $x $y)
312312macro_rules | `($x ^ $y) => `(rightact% HPow.hPow $x $y)
313313macro_rules | `($x ++ $y) => `(binop% HAppend.hAppend $x $y)
314314macro_rules | `(- $x) => `(unop% Neg.neg $x)
315- macro_rules | `($x ⁻¹) => `(unop% Inv.inv $x)
316315
317316recommended_spelling "or" for "|||" in [HOr.hOr, «term_|||_ »]
318317recommended_spelling "xor" for "^^^" in [HXor.hXor, «term_^^^_ »]
@@ -327,6 +326,7 @@ recommended_spelling "pow" for "^" in [HPow.hPow, «term_^_»]
327326recommended_spelling "append" for "++" in [HAppend.hAppend, «term_++_ »]
328327/-- when used as a unary operator -/
329328recommended_spelling "neg" for "-" in [Neg.neg, «term-_ »]
329+ recommended_spelling "inv" for "⁻¹" in [Inv.inv]
330330recommended_spelling "dvd" for "∣" in [Dvd.dvd, «term_∣_ »]
331331recommended_spelling "shiftLeft" for "<<<" in [HShiftLeft.hShiftLeft, «term_<<<_ »]
332332recommended_spelling "shiftRight" for ">>>" in [HShiftRight.hShiftRight, «term_>>>_ »]
0 commit comments