Skip to content

Commit

Permalink
chore: classify porting notes referring to missing linters (#12098)
Browse files Browse the repository at this point in the history
Reference the newly created issues #12094 and #12096, as well as the pre-existing #5171.
Change all references to #10927 to #5171.
Some of these changes were not labelled as "porting note"; change this for good measure.
  • Loading branch information
grunweg authored and Louddy committed Apr 15, 2024
1 parent 17614ee commit 637d8aa
Show file tree
Hide file tree
Showing 116 changed files with 201 additions and 174 deletions.
8 changes: 5 additions & 3 deletions Mathlib/Algebra/AddTorsor.lean
Expand Up @@ -53,13 +53,15 @@ class AddTorsor (G : outParam (Type*)) (P : Type*) [outParam <| AddGroup G] exte
vadd_vsub' : ∀ (g : G) (p : P), g +ᵥ p -ᵥ p = g
#align add_torsor AddTorsor

attribute [instance 100] AddTorsor.nonempty -- Porting note: removers `nolint instance_priority`
-- Porting note(#12096): removed `nolint instance_priority`; lint not ported yet
attribute [instance 100] AddTorsor.nonempty

-- Porting note: removed
-- Porting note(#12094): removed nolint; dangerous_instance linter not ported yet
--attribute [nolint dangerous_instance] AddTorsor.toVSub

/-- An `AddGroup G` is a torsor for itself. -/
--@[nolint instance_priority] Porting note: linter does not exist
-- Porting note(#12096): linter not ported yet
--@[nolint instance_priority]
instance addGroupIsAddTorsor (G : Type*) [AddGroup G] : AddTorsor G G
where
vsub := Sub.sub
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Algebra/Basic.lean
Expand Up @@ -105,7 +105,7 @@ section Prio
See the implementation notes in this file for discussion of the details of this definition.
-/
-- Porting note: unsupported @[nolint has_nonempty_instance]
-- Porting note(#5171): unsupported @[nolint has_nonempty_instance]
class Algebra (R : Type u) (A : Type v) [CommSemiring R] [Semiring A] extends SMul R A,
R →+* A where
commutes' : ∀ r x, toRingHom r * x = x * toRingHom r
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Algebra/Hom.lean
Expand Up @@ -28,7 +28,7 @@ open BigOperators
universe u v w u₁ v₁

/-- Defining the homomorphism in the category R-Alg. -/
-- @[nolint has_nonempty_instance] -- Porting note: This linter does not exist yet.
-- @[nolint has_nonempty_instance] -- Porting note(#5171): linter not ported yet
structure AlgHom (R : Type u) (A : Type v) (B : Type w) [CommSemiring R] [Semiring A] [Semiring B]
[Algebra R A] [Algebra R B] extends RingHom A B where
commutes' : ∀ r : R, toFun (algebraMap R A r) = algebraMap R B r
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Algebra/Tower.lean
Expand Up @@ -177,7 +177,7 @@ instance (priority := 999) subsemiring (U : Subsemiring S) : IsScalarTower U S A
of_algebraMap_eq fun _x => rfl
#align is_scalar_tower.subsemiring IsScalarTower.subsemiring

-- Porting note: @[nolint instance_priority]
-- Porting note(#12096): removed @[nolint instance_priority], linter not ported yet
instance (priority := 999) of_algHom {R A B : Type*} [CommSemiring R] [CommSemiring A]
[CommSemiring B] [Algebra R A] [Algebra R B] (f : A →ₐ[R] B) :
@IsScalarTower R A B _ f.toRingHom.toAlgebra.toSMul _ :=
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean
Expand Up @@ -238,7 +238,7 @@ universe v u
we will equip with a category structure where the morphisms are formal `R`-linear combinations
of the morphisms in `C`.
-/
-- Porting note: Removed has_nonempty_instance nolint
-- Porting note(#5171): Removed has_nonempty_instance nolint; linter not ported yet
@[nolint unusedArguments]
def Free (_ : Type*) (C : Type u) :=
C
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Homology/Homotopy.lean
Expand Up @@ -130,7 +130,7 @@ theorem prevD_nat (C D : CochainComplex V ℕ) (i : ℕ) (f : ∀ i j, C.X i ⟶
· congr <;> simp
#align prev_d_nat prevD_nat

-- Porting note: removed @[has_nonempty_instance]
-- Porting note(#5171): removed @[has_nonempty_instance]
/-- A homotopy `h` between chain maps `f` and `g` consists of components `h i j : C.X i ⟶ D.X j`
which are zero unless `c.Rel j i`, satisfying the homotopy condition.
-/
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Module/LocalizedModule.lean
Expand Up @@ -77,7 +77,7 @@ example {R} [CommSemiring R] (S : Submonoid R) : ⇑(Localization.r' S) = Locali
/-- If `S` is a multiplicative subset of a ring `R` and `M` an `R`-module, then
we can localize `M` by `S`.
-/
-- Porting note: @[nolint has_nonempty_instance]
-- Porting note(#5171): @[nolint has_nonempty_instance]
def _root_.LocalizedModule : Type max u v :=
Quotient (r.setoid S M)
#align localized_module LocalizedModule
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Algebra/Order/Group/Cone.lean
Expand Up @@ -24,7 +24,7 @@ namespace AddCommGroup
/-- A collection of elements in an `AddCommGroup` designated as "non-negative".
This is useful for constructing an `OrderedAddCommGroup`
by choosing a positive cone in an existing `AddCommGroup`. -/
-- Porting note: @[nolint has_nonempty_instance]
-- Porting note(#5171): @[nolint has_nonempty_instance]
structure PositiveCone (α : Type*) [AddCommGroup α] where
/-- The characteristic predicate of a positive cone. `nonneg a` means that `0 ≤ a` according to
the cone. -/
Expand All @@ -40,7 +40,7 @@ structure PositiveCone (α : Type*) [AddCommGroup α] where

/-- A positive cone in an `AddCommGroup` induces a linear order if
for every `a`, either `a` or `-a` is non-negative. -/
-- Porting note: @[nolint has_nonempty_instance]
-- Porting note(#5171): @[nolint has_nonempty_instance]
structure TotalPositiveCone (α : Type*) [AddCommGroup α] extends PositiveCone α where
/-- For any `a` the proposition `nonneg a` is decidable -/
nonnegDecidable : DecidablePred nonneg
Expand Down
3 changes: 2 additions & 1 deletion Mathlib/Algebra/Ring/CompTypeclasses.lean
Expand Up @@ -179,7 +179,8 @@ theorem RingHom.surjective (σ : R₁ →+* R₂) [t : RingHomSurjective σ] : F
namespace RingHomSurjective

-- The linter gives a false positive, since `σ₂` is an out_param
-- @[nolint dangerous_instance] Porting note: this linter is not implemented yet
-- Porting note(#12094): removed nolint; dangerous_instance linter not ported yet
-- @[nolint dangerous_instance]
instance (priority := 100) invPair {σ₁ : R₁ →+* R₂} {σ₂ : R₂ →+* R₁} [RingHomInvPair σ₁ σ₂] :
RingHomSurjective σ₁ :=
fun x => ⟨σ₂ x, RingHomInvPair.comp_apply_eq₂⟩⟩
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Star/CHSH.lean
Expand Up @@ -82,7 +82,7 @@ the `Aᵢ` commute with the `Bⱼ`.
The physical interpretation is that `A₀` and `A₁` are a pair of boolean observables which
are spacelike separated from another pair `B₀` and `B₁` of boolean observables.
-/
--@[nolint has_nonempty_instance] Porting note: linter does not exist
--@[nolint has_nonempty_instance] Porting note(#5171): linter not ported yet
structure IsCHSHTuple {R} [Monoid R] [StarMul R] (A₀ A₁ B₀ B₁ : R) : Prop where
A₀_inv : A₀ ^ 2 = 1
A₁_inv : A₁ ^ 2 = 1
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/AlgebraicGeometry/AffineScheme.lean
Expand Up @@ -45,7 +45,7 @@ namespace AlgebraicGeometry
open Spec (structureSheaf)

/-- The category of affine schemes -/
-- Porting note: removed
-- Porting note(#5171): linter not ported yet
-- @[nolint has_nonempty_instance]
def AffineScheme :=
Scheme.Spec.EssImageSubcategory
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/AlgebraicGeometry/Gluing.lean
Expand Up @@ -82,7 +82,7 @@ such that
We can then glue the schemes `U i` together by identifying `V i j` with `V j i`, such
that the `U i`'s are open subschemes of the glued space.
-/
-- Porting note: @[nolint has_nonempty_instance]
-- Porting note(#5171): @[nolint has_nonempty_instance]; linter not ported yet
structure GlueData extends CategoryTheory.GlueData Scheme where
f_open : ∀ i j, IsOpenImmersion (f i j)
#align algebraic_geometry.Scheme.glue_data AlgebraicGeometry.Scheme.GlueData
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Topology.lean
Expand Up @@ -46,7 +46,7 @@ variable {R A : Type*}
variable [CommSemiring R] [CommRing A] [Algebra R A]
variable (𝒜 : ℕ → Submodule R A) [GradedAlgebra 𝒜]

-- porting note (#10927): removed @[nolint has_nonempty_instance]
-- porting note (#5171): removed @[nolint has_nonempty_instance]
/-- The projective spectrum of a graded commutative ring is the subtype of all homogenous ideals
that are prime and do not contain the irrelevant ideal. -/
@[ext]
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/AlgebraicGeometry/Scheme.lean
Expand Up @@ -49,7 +49,7 @@ structure Scheme extends LocallyRingedSpace where
namespace Scheme

/-- A morphism between schemes is a morphism between the underlying locally ringed spaces. -/
-- @[nolint has_nonempty_instance] -- Porting note: no such linter.
-- @[nolint has_nonempty_instance] -- Porting note(#5171): linter not ported yet
def Hom (X Y : Scheme) : Type* :=
X.toLocallyRingedSpace ⟶ Y.toLocallyRingedSpace
#align algebraic_geometry.Scheme.hom AlgebraicGeometry.Scheme.Hom
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/AlgebraicTopology/DoldKan/Decomposition.lean
Expand Up @@ -84,7 +84,7 @@ set_option linter.uppercaseLean3 false in

variable (X)

-- porting note (#10927): removed @[nolint has_nonempty_instance]
-- porting note (#5171): removed @[nolint has_nonempty_instance]
/-- The structure `MorphComponents` is an ad hoc structure that is used in
the proof that `N₁ : SimplicialObject C ⥤ Karoubi (ChainComplex C ℕ))`
reflects isomorphisms. The fields are the data that are needed in order to
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/AlgebraicTopology/SimplexCategory.lean
Expand Up @@ -89,7 +89,7 @@ protected def rec {F : SimplexCategory → Sort*} (h : ∀ n : ℕ, F [n]) : ∀
h n.len
#align simplex_category.rec SimplexCategory.rec

-- porting note (#10927): removed @[nolint has_nonempty_instance]
-- porting note (#5171): removed @[nolint has_nonempty_instance]
/-- Morphisms in the `SimplexCategory`. -/
protected def Hom (a b : SimplexCategory) :=
Fin (a.len + 1) →o Fin (b.len + 1)
Expand Down
12 changes: 6 additions & 6 deletions Mathlib/AlgebraicTopology/SimplicialObject.lean
Expand Up @@ -33,7 +33,7 @@ namespace CategoryTheory

variable (C : Type u) [Category.{v} C]

-- porting note (#10927): removed @[nolint has_nonempty_instance]
-- porting note (#5171): removed @[nolint has_nonempty_instance]
/-- The category of simplicial objects valued in a category `C`.
This is the category of contravariant functors from `SimplexCategory` to `C`. -/
def SimplicialObject :=
Expand Down Expand Up @@ -224,7 +224,7 @@ def whiskering (D : Type*) [Category D] : (C ⥤ D) ⥤ SimplicialObject C ⥤ S
whiskeringRight _ _ _
#align category_theory.simplicial_object.whiskering CategoryTheory.SimplicialObject.whiskering

-- porting note (#10927): removed @[nolint has_nonempty_instance]
-- porting note (#5171): removed @[nolint has_nonempty_instance]
/-- Truncated simplicial objects. -/
def Truncated (n : ℕ) :=
(SimplexCategory.Truncated n)ᵒᵖ ⥤ C
Expand Down Expand Up @@ -282,7 +282,7 @@ abbrev const : C ⥤ SimplicialObject C :=
CategoryTheory.Functor.const _
#align category_theory.simplicial_object.const CategoryTheory.SimplicialObject.const

-- porting note (#10927): removed @[nolint has_nonempty_instance]
-- porting note (#5171): removed @[nolint has_nonempty_instance]
/-- The category of augmented simplicial objects, defined as a comma category. -/
def Augmented :=
Comma (𝟭 (SimplicialObject C)) (const C)
Expand Down Expand Up @@ -403,7 +403,7 @@ theorem augment_hom_zero (X : SimplicialObject C) (X₀ : C) (f : X _[0] ⟶ X

end SimplicialObject

-- porting note (#10927): removed @[nolint has_nonempty_instance]
-- porting note (#5171): removed @[nolint has_nonempty_instance]
/-- Cosimplicial objects. -/
def CosimplicialObject :=
SimplexCategory ⥤ C
Expand Down Expand Up @@ -593,7 +593,7 @@ def whiskering (D : Type*) [Category D] : (C ⥤ D) ⥤ CosimplicialObject C ⥤
whiskeringRight _ _ _
#align category_theory.cosimplicial_object.whiskering CategoryTheory.CosimplicialObject.whiskering

-- porting note (#10927): removed @[nolint has_nonempty_instance]
-- porting note (#5171): removed @[nolint has_nonempty_instance]
/-- Truncated cosimplicial objects. -/
def Truncated (n : ℕ) :=
SimplexCategory.Truncated n ⥤ C
Expand Down Expand Up @@ -651,7 +651,7 @@ abbrev const : C ⥤ CosimplicialObject C :=
CategoryTheory.Functor.const _
#align category_theory.cosimplicial_object.const CategoryTheory.CosimplicialObject.const

-- porting note (#10927): removed @[nolint has_nonempty_instance]
-- porting note (#5171): removed @[nolint has_nonempty_instance]
/-- Augmented cosimplicial objects. -/
def Augmented :=
Comma (const C) (𝟭 (CosimplicialObject C))
Expand Down
6 changes: 3 additions & 3 deletions Mathlib/AlgebraicTopology/SplitSimplicialObject.lean
Expand Up @@ -214,7 +214,7 @@ def cofan' (Δ : SimplexCategoryᵒᵖ) : Cofan (summand N Δ) :=

end Splitting

--porting note (#10927): removed @[nolint has_nonempty_instance]
--porting note (#5171): removed @[nolint has_nonempty_instance]
/-- A splitting of a simplicial object `X` consists of the datum of a sequence
of objects `N`, a sequence of morphisms `ι : N n ⟶ X _[n]` such that
for all `Δ : SimplexCategoryᵒᵖ`, the canonical map `Splitting.map X ι Δ`
Expand Down Expand Up @@ -314,7 +314,7 @@ end Splitting

variable (C)

-- porting note (#10927): removed @[nolint has_nonempty_instance]
-- porting note (#5171): removed @[nolint has_nonempty_instance]
/-- The category `SimplicialObject.Split C` is the category of simplicial objects
in `C` equipped with a splitting, and morphisms are morphisms of simplicial objects
which are compatible with the splittings. -/
Expand All @@ -337,7 +337,7 @@ def mk' {X : SimplicialObject C} (s : Splitting X) : Split C :=
⟨X, s⟩
#align simplicial_object.split.mk' SimplicialObject.Split.mk'

-- porting note (#10927): removed @[nolint has_nonempty_instance]
-- porting note (#5171): removed @[nolint has_nonempty_instance]
/-- Morphisms in `SimplicialObject.Split C` are morphisms of simplicial objects that
are compatible with the splittings. -/
structure Hom (S₁ S₂ : Split C) where
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Analysis/Calculus/BumpFunction/Basic.lean
Expand Up @@ -82,7 +82,7 @@ add more properties if they are useful and satisfied in the examples of inner pr
and finite dimensional vector spaces, notably derivative norm control in terms of `R - 1`.
TODO: do we ever need `f x = 1 ↔ ‖x‖ ≤ 1`? -/
-- Porting note: was @[nolint has_nonempty_instance]
-- Porting note(#5171): linter not yet ported; was @[nolint has_nonempty_instance]
structure ContDiffBumpBase (E : Type*) [NormedAddCommGroup E] [NormedSpace ℝ E] where
toFun : ℝ → E → ℝ
mem_Icc : ∀ (R : ℝ) (x : E), toFun R x ∈ Icc (0 : ℝ) 1
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Analysis/Calculus/Implicit.lean
Expand Up @@ -96,7 +96,7 @@ needs to have a complete control over the choice of the implicit function.
* both functions are strictly differentiable at `a`;
* the derivatives are surjective;
* the kernels of the derivatives are complementary subspaces of `E`. -/
-- Porting note: not yet supported @[nolint has_nonempty_instance]
-- Porting note(#5171): linter not yet ported @[nolint has_nonempty_instance]
structure ImplicitFunctionData (𝕜 : Type*) [NontriviallyNormedField 𝕜] (E : Type*)
[NormedAddCommGroup E] [NormedSpace 𝕜 E] [CompleteSpace E] (F : Type*) [NormedAddCommGroup F]
[NormedSpace 𝕜 F] [CompleteSpace F] (G : Type*) [NormedAddCommGroup G] [NormedSpace 𝕜 G]
Expand Down
3 changes: 2 additions & 1 deletion Mathlib/Analysis/RCLike/Lemmas.lean
Expand Up @@ -34,7 +34,8 @@ This instance generates a type-class problem with a metavariable `?m` that shoul
`RCLike ?m`. Since this can only be satisfied by `ℝ` or `ℂ`, this does not cause problems. -/

/-- An `RCLike` field is finite-dimensional over `ℝ`, since it is spanned by `{1, I}`. -/
-- Porting note: was @[nolint dangerous_instance]
-- Porting note(#12094): removed nolint; dangerous_instance linter not ported yet
-- @[nolint dangerous_instance]
instance rclike_to_real : FiniteDimensional ℝ K :=
⟨{1, I}, by
suffices ∀ x : K, ∃ a b : ℝ, a • 1 + b • I = x by
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/CategoryTheory/Adjunction/Basic.lean
Expand Up @@ -242,7 +242,7 @@ namespace Adjunction
See `Adjunction.mkOfHomEquiv`.
This structure won't typically be used anywhere else.
-/
-- Porting comment: `has_nonempty_instance` linter doesn't exist (yet?)
-- Porting note(#5171): `has_nonempty_instance` linter not ported yet
-- @[nolint has_nonempty_instance]
structure CoreHomEquiv (F : C ⥤ D) (G : D ⥤ C) where
/-- The equivalence between `Hom (F X) Y` and `Hom X (G Y)` -/
Expand Down Expand Up @@ -304,7 +304,7 @@ end CoreHomEquiv
See `Adjunction.mkOfUnitCounit`.
This structure won't typically be used anywhere else.
-/
-- Porting comment: `has_nonempty_instance` linter doesn't exist (yet?)
-- Porting note(#5171): `has_nonempty_instance` linter not ported yet
-- @[nolint has_nonempty_instance]
structure CoreUnitCounit (F : C ⥤ D) (G : D ⥤ C) where
/-- The unit of an adjunction between `F` and `G` -/
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Bicategory/Free.lean
Expand Up @@ -64,7 +64,7 @@ instance categoryStruct : CategoryStruct.{max u v} (FreeBicategory B) where
comp := @fun _ _ _ => Hom.comp

/-- Representatives of 2-morphisms in the free bicategory. -/
-- Porting note: no such linter
-- Porting note(#5171): linter not ported yet
-- @[nolint has_nonempty_instance]
inductive Hom₂ : ∀ {a b : FreeBicategory B}, (a ⟶ b) → (a ⟶ b) → Type max u v
| id {a b} (f : a ⟶ b) : Hom₂ f f
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/CategoryTheory/Bicategory/Functor.lean
Expand Up @@ -313,8 +313,8 @@ def comp (F : OplaxFunctor B C) (G : OplaxFunctor C D) : OplaxFunctor B D :=
/-- A structure on an oplax functor that promotes an oplax functor to a pseudofunctor.
See `Pseudofunctor.mkOfOplax`.
-/
-- Porting note: removing no lint for nonempty_instance
--@[nolint has_nonempty_instance]
-- Porting note(#5171): linter not ported yet
-- @[nolint has_nonempty_instance]
-- Porting note: removing primes in structure name because
-- my understanding is that they're no longer needed
structure PseudoCore (F : OplaxFunctor B C) where
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Category/PartialFun.lean
Expand Up @@ -45,7 +45,7 @@ namespace PartialFun
instance : CoeSort PartialFun (Type*) :=
⟨id⟩

-- Porting note: removed `@[nolint has_nonempty_instance]`
-- Porting note(#5171): removed `@[nolint has_nonempty_instance]`; linter not ported yet
/-- Turns a type into a `PartialFun`. -/
def of : Type* → PartialFun :=
id
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/CommSq.lean
Expand Up @@ -108,7 +108,7 @@ variable {A B X Y : C} {f : A ⟶ X} {i : A ⟶ B} {p : X ⟶ Y} {g : B ⟶ Y}
The datum of a lift in a commutative square, i.e. an up-right-diagonal
morphism which makes both triangles commute. -/
-- porting note (#10927): removed @[nolint has_nonempty_instance]
-- porting note (#5171): removed @[nolint has_nonempty_instance]
@[ext]
structure LiftStruct (sq : CommSq f i p g) where
/-- The lift. -/
Expand Down
3 changes: 2 additions & 1 deletion Mathlib/CategoryTheory/Comma/StructuredArrow.lean
Expand Up @@ -36,6 +36,7 @@ and morphisms `C`-morphisms `Y ⟶ Y'` making the obvious triangle commute.
-/
-- We explicitly come from `PUnit.{1}` here to obtain the correct universe for morphisms of
-- structured arrows.
-- Porting note(#5171): linter not ported yet
-- @[nolint has_nonempty_instance]
def StructuredArrow (S : D) (T : C ⥤ D) :=
Comma (Functor.fromPUnit.{0} S) T
Expand Down Expand Up @@ -380,7 +381,7 @@ and morphisms `C`-morphisms `Y ⟶ Y'` making the obvious triangle commute.
-/
-- We explicitly come from `PUnit.{1}` here to obtain the correct universe for morphisms of
-- costructured arrows.
-- @[nolint has_nonempty_instance] -- Porting note: removed
-- @[nolint has_nonempty_instance] -- Porting note(#5171): linter not ported yet
def CostructuredArrow (S : C ⥤ D) (T : D) :=
Comma S (Functor.fromPUnit.{0} T)
#align category_theory.costructured_arrow CategoryTheory.CostructuredArrow
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/CategoryTheory/Core.lean
Expand Up @@ -30,7 +30,7 @@ universe v₁ v₂ u₁ u₂
-- morphism levels before object levels. See note [CategoryTheory universes].
/-- The core of a category C is the groupoid whose morphisms are all the
isomorphisms of C. -/
-- Porting note: This linter does not exist yet
-- Porting note(#5171): linter not yet ported
-- @[nolint has_nonempty_instance]

def Core (C : Type u₁) := C
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/CategoryTheory/DifferentialObject.lean
Expand Up @@ -35,7 +35,7 @@ variable [HasZeroMorphisms C] [HasShift C S]
/-- A differential object in a category with zero morphisms and a shift is
an object `obj` equipped with
a morphism `d : obj ⟶ obj⟦1⟧`, such that `d^2 = 0`. -/
-- Porting note: Removed `@[nolint has_nonempty_instance]`
-- Porting note(#5171): removed `@[nolint has_nonempty_instance]`
structure DifferentialObject where
/-- The underlying object of a differential object. -/
obj : C
Expand All @@ -54,7 +54,7 @@ variable {S C}
namespace DifferentialObject

/-- A morphism of differential objects is a morphism commuting with the differentials. -/
@[ext] -- Porting note: Removed `nolint has_nonempty_instance`
@[ext] -- Porting note(#5171): removed `nolint has_nonempty_instance`
structure Hom (X Y : DifferentialObject S C) where
/-- The morphism between underlying objects of the two differentiable objects. -/
f : X.obj ⟶ Y.obj
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/CategoryTheory/Enriched/Basic.lean
Expand Up @@ -172,7 +172,7 @@ section

variable {W : Type (v + 1)} [Category.{v} W] [MonoidalCategory W] [EnrichedCategory W C]

-- Porting note: removed `@[nolint has_nonempty_instance]`
-- Porting note(#5171): removed `@[nolint has_nonempty_instance]`
/-- A type synonym for `C`, which should come equipped with a `V`-enriched category structure.
In a moment we will equip this with the (honest) category structure
so that `X ⟶ Y` is `(𝟙_ W) ⟶ (X ⟶[W] Y)`.
Expand Down Expand Up @@ -391,7 +391,7 @@ coming from the ambient braiding on `V`.)
-/


-- Porting note: removed `@[nolint has_nonempty_instance]`
-- Porting note(#5171): removed `@[nolint has_nonempty_instance]`
/-- The type of `A`-graded natural transformations between `V`-functors `F` and `G`.
This is the type of morphisms in `V` from `A` to the `V`-object of natural transformations.
-/
Expand Down

0 comments on commit 637d8aa

Please sign in to comment.