Skip to content

Commit abc85c2

Browse files
authored
chore: fix Inv.inv notation (#8351)
1 parent 4362219 commit abc85c2

File tree

2 files changed

+4
-4
lines changed

2 files changed

+4
-4
lines changed

src/Init/Notation.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -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)
312312
macro_rules | `($x ^ $y) => `(rightact% HPow.hPow $x $y)
313313
macro_rules | `($x ++ $y) => `(binop% HAppend.hAppend $x $y)
314314
macro_rules | `(- $x) => `(unop% Neg.neg $x)
315-
macro_rules | `($x ⁻¹) => `(unop% Inv.inv $x)
316315

317316
recommended_spelling "or" for "|||" in [HOr.hOr, «term_|||_»]
318317
recommended_spelling "xor" for "^^^" in [HXor.hXor, «term_^^^_»]
@@ -327,6 +326,7 @@ recommended_spelling "pow" for "^" in [HPow.hPow, «term_^_»]
327326
recommended_spelling "append" for "++" in [HAppend.hAppend, «term_++_»]
328327
/-- when used as a unary operator -/
329328
recommended_spelling "neg" for "-" in [Neg.neg, «term-_»]
329+
recommended_spelling "inv" for "⁻¹" in [Inv.inv]
330330
recommended_spelling "dvd" for "∣" in [Dvd.dvd, «term_∣_»]
331331
recommended_spelling "shiftLeft" for "<<<" in [HShiftLeft.hShiftLeft, «term_<<<_»]
332332
recommended_spelling "shiftRight" for ">>>" in [HShiftRight.hShiftRight, «term_>>>_»]

src/Init/Prelude.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1661,7 +1661,7 @@ instance instAddNat : Add Nat where
16611661

16621662
/- We mark the following definitions as pattern to make sure they can be used in recursive equations,
16631663
and reduced by the equation Compiler. -/
1664-
attribute [match_pattern] Nat.add Add.add HAdd.hAdd Neg.neg Mul.mul HMul.hMul
1664+
attribute [match_pattern] Nat.add Add.add HAdd.hAdd Neg.neg Mul.mul HMul.hMul Inv.inv
16651665

16661666
set_option bootstrap.genMatcherCode false in
16671667
/--

0 commit comments

Comments
 (0)