Skip to content

Commit

Permalink
chore: classify new definition porting notes (#11512)
Browse files Browse the repository at this point in the history
Classifies by adding issue number #11446 to porting notes claiming "added definition".
  • Loading branch information
pitmonticone authored and utensil committed Mar 26, 2024
1 parent aa68106 commit 79fb032
Show file tree
Hide file tree
Showing 4 changed files with 4 additions and 4 deletions.
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Lie/UniversalEnveloping.lean
Original file line number Diff line number Diff line change
Expand Up @@ -88,7 +88,7 @@ def mkAlgHom : TensorAlgebra R L →ₐ[R] UniversalEnvelopingAlgebra R L :=
variable {L}

/-- The natural Lie algebra morphism from a Lie algebra to its universal enveloping algebra. -/
@[simps!] -- Porting note: added
@[simps!] -- Porting note (#11445): added
def ι : L →ₗ⁅R⁆ UniversalEnvelopingAlgebra R L :=
{ (mkAlgHom R L).toLinearMap.comp ιₜ with
map_lie' := fun {x y} => by
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Sites/Grothendieck.lean
Original file line number Diff line number Diff line change
Expand Up @@ -424,7 +424,7 @@ instance : Coe (J.Cover X) (Sieve X) :=
-/

/-
Porting note: Added this def as a replacement for the "dangerous" `Coe` above.
Porting note (#11445): Added this def as a replacement for the "dangerous" `Coe` above.
-/
/-- The sieve associated to a term of `J.Cover X`.-/
def sieve (S : J.Cover X) : Sieve X := S.1
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/NumberTheory/ArithmeticFunction.lean
Original file line number Diff line number Diff line change
Expand Up @@ -837,7 +837,7 @@ end IsMultiplicative
section SpecialFunctions

/-- The identity on `ℕ` as an `ArithmeticFunction`. -/
nonrec -- Porting note: added
nonrec -- Porting note (#11445): added
def id : ArithmeticFunction ℕ :=
⟨id, rfl⟩
#align nat.arithmetic_function.id ArithmeticFunction.id
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/SetTheory/Game/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -49,7 +49,7 @@ abbrev Game :=

namespace Game

-- Porting note: added this definition
-- Porting note (#11445): added this definition
/-- Negation of games. -/
instance : Neg Game where
neg := Quot.map Neg.neg <| fun _ _ => (neg_equiv_neg_iff).2
Expand Down

0 comments on commit 79fb032

Please sign in to comment.