Skip to content

Commit

Permalink
chore: classify new definition porting notes (#11446)
Browse files Browse the repository at this point in the history
Classifies by adding issue number #11445 to porting notes claiming anything equivalent to: 

- "new definition"
- "added definition"
  • Loading branch information
pitmonticone committed Mar 17, 2024
1 parent 15ca3da commit 3fcb743
Show file tree
Hide file tree
Showing 9 changed files with 12 additions and 12 deletions.
6 changes: 3 additions & 3 deletions Mathlib/Algebra/Algebra/Hom.lean
Expand Up @@ -69,7 +69,7 @@ instance (priority := 100) linearMapClass [AlgHomClass F R A B] : LinearMapClass
simp only [Algebra.smul_def, map_mul, commutes, RingHom.id_apply] }
#align alg_hom_class.linear_map_class AlgHomClass.linearMapClass

-- Porting note: A new definition underlying a coercion `↑`.
-- Porting note (#11445): A new definition underlying a coercion `↑`.
/-- Turn an element of a type `F` satisfying `AlgHomClass F α β` into an actual
`AlgHom`. This is declared as the default coercion from `F` to `α →+* β`. -/
@[coe]
Expand Down Expand Up @@ -132,15 +132,15 @@ theorem toFun_eq_coe (f : A →ₐ[R] B) : f.toFun = f :=

#noalign alg_hom.coe_ring_hom

-- Porting note: A new definition underlying a coercion `↑`.
-- Porting note (#11445): A new definition underlying a coercion `↑`.
@[coe]
def toMonoidHom' (f : A →ₐ[R] B) : A →* B := (f : A →+* B)

instance coeOutMonoidHom : CoeOut (A →ₐ[R] B) (A →* B) :=
⟨AlgHom.toMonoidHom'⟩
#align alg_hom.coe_monoid_hom AlgHom.coeOutMonoidHom

-- Porting note: A new definition underlying a coercion `↑`.
-- Porting note (#11445): A new definition underlying a coercion `↑`.
@[coe]
def toAddMonoidHom' (f : A →ₐ[R] B) : A →+ B := (f : A →+* B)

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Analysis/NormedSpace/BoundedLinearMaps.lean
Expand Up @@ -355,7 +355,7 @@ theorem ContinuousLinearMap.isBoundedBilinearMap (f : E →L[𝕜] F →L[𝕜]
apply_rules [mul_le_mul_of_nonneg_right, norm_nonneg, le_max_left] ⟩ }
#align continuous_linear_map.is_bounded_bilinear_map ContinuousLinearMap.isBoundedBilinearMap

-- Porting note: new definition
-- Porting note (#11445): new definition
/-- A bounded bilinear map `f : E × F → G` defines a continuous linear map
`f : E →L[𝕜] F →L[𝕜] G`. -/
def IsBoundedBilinearMap.toContinuousLinearMap (hf : IsBoundedBilinearMap 𝕜 f) :
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Data/Complex/Exponential.lean
Expand Up @@ -195,7 +195,7 @@ theorem exp_add : exp (x + y) = exp x * exp y := by
exact cauchy_product (isCauSeq_abs_exp x) (isCauSeq_exp y)
#align complex.exp_add Complex.exp_add

-- Porting note: New definition
-- Porting note (#11445): new definition
/-- the exponential function as a monoid hom from `Multiplicative ℂ` to `ℂ` -/
noncomputable def expMonoidHom : MonoidHom (Multiplicative ℂ) ℂ :=
{ toFun := fun z => exp (Multiplicative.toAdd z),
Expand Down Expand Up @@ -816,7 +816,7 @@ theorem exp_zero : exp 0 = 1 := by simp [Real.exp]
nonrec theorem exp_add : exp (x + y) = exp x * exp y := by simp [exp_add, exp]
#align real.exp_add Real.exp_add

-- Porting note: New definition
-- Porting note (#11445): new definition
/-- the exponential function as a monoid hom from `Multiplicative ℝ` to `ℝ` -/
noncomputable def expMonoidHom : MonoidHom (Multiplicative ℝ) ℝ :=
{ toFun := fun x => exp (Multiplicative.toAdd x),
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/ENat/Basic.lean
Expand Up @@ -121,7 +121,7 @@ theorem toNat_top : toNat ⊤ = 0 :=

@[simp] theorem toNat_eq_zero : toNat n = 0 ↔ n = 0 ∨ n = ⊤ := WithTop.untop'_eq_self_iff

-- Porting note: new definition copied from `WithTop`
-- Porting note (#11445): new definition copied from `WithTop`
/-- Recursor for `ENat` using the preferred forms `⊤` and `↑a`. -/
@[elab_as_elim]
def recTopCoe {C : ℕ∞ → Sort*} (top : C ⊤) (coe : ∀ a : ℕ, C a) : ∀ n : ℕ∞, C n
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/Finset/Basic.lean
Expand Up @@ -200,7 +200,7 @@ instance decidableMem [_h : DecidableEq α] (a : α) (s : Finset α) : Decidable

/-! ### set coercion -/

-- Porting note: new definition
-- Porting note (#11445): new definition
/-- Convert a finset to a set in the natural way. -/
@[coe] def toSet (s : Finset α) : Set α :=
{ a | a ∈ s }
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/List/Cycle.lean
Expand Up @@ -453,7 +453,7 @@ namespace Cycle

variable {α : Type*}

-- Porting note: new definition
-- Porting note (#11445): new definition
/-- The coercion from `List α` to `Cycle α` -/
@[coe] def ofList : List α → Cycle α :=
Quot.mk _
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/PNat/Prime.lean
Expand Up @@ -18,7 +18,7 @@ This file extends the theory of `ℕ+` with `gcd`, `lcm` and `Prime` functions,

namespace Nat.Primes

-- Porting note: new definition
-- Porting note (#11445): new definition
/-- The canonical map from `Nat.Primes` to `ℕ+` -/
@[coe] def toPNat : Nat.Primes → ℕ+ :=
fun p => ⟨(p : ℕ), p.property.pos⟩
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/Sym/Basic.lean
Expand Up @@ -43,7 +43,7 @@ def Sym (α : Type*) (n : ℕ) :=
{ s : Multiset α // Multiset.card s = n }
#align sym Sym

-- Porting note: new definition
-- Porting note (#11445): new definition
/-- The canonical map to `Multiset α` that forgets that `s` has length `n` -/
@[coe] def Sym.toMultiset {α : Type*} {n : ℕ} (s : Sym α n) : Multiset α :=
s.1
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/ModelTheory/Basic.lean
Expand Up @@ -365,7 +365,7 @@ scoped[FirstOrder] notation:25 A " ≃[" L "] " B => FirstOrder.Language.Equiv L
-- The former reported an error.
variable {L M N} {P : Type*} [Structure L P] {Q : Type*} [Structure L Q]

-- Porting note: new definition
-- Porting note (#11445): new definition
/-- Interpretation of a constant symbol -/
@[coe]
def constantMap (c : L.Constants) : M := funMap c default
Expand Down

0 comments on commit 3fcb743

Please sign in to comment.