Skip to content

Commit

Permalink
chore: classify removed @[pp_nodot] porting notes (#11181)
Browse files Browse the repository at this point in the history
Classifies by adding issue number #11180 to porting notes claiming: 

> removed `@[pp_nodot]`
  • Loading branch information
pitmonticone authored and kbuzzard committed Mar 12, 2024
1 parent b55aaee commit c30fa3d
Show file tree
Hide file tree
Showing 3 changed files with 4 additions and 4 deletions.
4 changes: 2 additions & 2 deletions Mathlib/Algebra/Symmetrized.lean
Original file line number Diff line number Diff line change
Expand Up @@ -47,13 +47,13 @@ variable {α : Type*}

/-- The element of `SymAlg α` that represents `a : α`. -/
@[match_pattern]
-- Porting note: removed @[pp_nodot]
-- Porting note (#11180): removed @[pp_nodot]
def sym : α ≃ αˢʸᵐ :=
Equiv.refl _
#align sym_alg.sym SymAlg.sym

/-- The element of `α` represented by `x : αˢʸᵐ`. -/
-- Porting note: removed @[pp_nodot]
-- Porting note (#11180): removed @[pp_nodot]
def unsym : αˢʸᵐ ≃ α :=
Equiv.refl _
#align sym_alg.unsym SymAlg.unsym
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/Nat/Prime.lean
Original file line number Diff line number Diff line change
Expand Up @@ -43,7 +43,7 @@ variable {n : ℕ}

/-- `Nat.Prime p` means that `p` is a prime number, that is, a natural number
at least 2 whose only divisors are `p` and `1`. -/
-- Porting note: removed @[pp_nodot]
-- Porting note (#11180): removed @[pp_nodot]
def Prime (p : ℕ) :=
Irreducible p
#align nat.prime Nat.Prime
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/Real/NNReal.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1155,7 +1155,7 @@ end Set
namespace Real

/-- The absolute value on `ℝ` as a map to `ℝ≥0`. -/
-- Porting note: removed @[pp_nodot]
-- Porting note (#11180): removed @[pp_nodot]
def nnabs : ℝ →*₀ ℝ≥0 where
toFun x := ⟨|x|, abs_nonneg x⟩
map_zero' := by ext; simp
Expand Down

0 comments on commit c30fa3d

Please sign in to comment.