Skip to content

Commit

Permalink
wip
Browse files Browse the repository at this point in the history
  • Loading branch information
joelriou committed Dec 27, 2024
1 parent bebe433 commit 8b9474e
Show file tree
Hide file tree
Showing 2 changed files with 29 additions and 2 deletions.
Original file line number Diff line number Diff line change
Expand Up @@ -37,6 +37,9 @@ variable {X : C} {κ : Cardinal.{w}} [Fact κ.IsRegular]

variable (p : CardinalFilteredPresentation X κ)

instance isFiltered : IsFiltered p.J := by
apply isFiltered_of_isCardinalDirected _ κ

lemma isCardinalPresentable_pt (h : ∀ (j : p.J), IsCardinalPresentable (p.F.obj j) κ)
[LocallySmall.{w} C]
(κ' : Cardinal.{w}) [Fact κ'.IsRegular] (h : κ ≤ κ')
Expand Down
28 changes: 26 additions & 2 deletions Mathlib/CategoryTheory/Presentable/Comma.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,6 +6,7 @@ Authors: Joël Riou

import Mathlib.CategoryTheory.Presentable.LocallyPresentable
import Mathlib.CategoryTheory.Limits.Comma
import Mathlib.CategoryTheory.Limits.Final
import Mathlib.CategoryTheory.Comma.LocallySmall

/-!
Expand All @@ -28,9 +29,12 @@ variable (κ : Cardinal.{w}) [Fact κ.IsRegular]

variable {F₁ F₂} in
instance isCardinalPresentable_mk {X₁ : C₁} {X₂ : C₂}
[IsCardinalPresentable X₁ κ] [IsCardinalPresentable X₂ κ]
[IsCardinalPresentable X₁ κ] [IsCardinalPresentable X₂ κ]
(f : F₁.obj X₁ ⟶ F₂.obj X₂) :
IsCardinalPresentable (Comma.mk _ _ f) κ := sorry
IsCardinalPresentable (Comma.mk _ _ f) κ := by
-- need that `F₁` (and `F₂` ?) preserve κ-presentable objects
sorry

section

Expand Down Expand Up @@ -100,6 +104,18 @@ variable {S₁ S₂ S₃ : Index f p₁ p₂} (φ : S₁ ⟶ S₂) (φ' : S₂

end

variable (f p₁ p₂)

@[simps]
def π₁ : Index f p₁ p₂ ⥤ p₁.J where
obj S := S.j₁
map φ := φ.m₁

@[simps]
def π₂ : Index f p₁ p₂ ⥤ p₂.J where
obj S := S.j₂
map φ := φ.m₂

end Index

@[simps]
Expand Down Expand Up @@ -137,13 +153,21 @@ instance [LocallySmall.{w} D] : EssentiallySmall.{w} (Index f p₁ p₂) := by

instance : IsCardinalFiltered (Index f p₁ p₂) κ := sorry

instance : IsFiltered (Index f p₁ p₂) := by
apply isFiltered_of_isCardinalDirected _ κ

instance : (Index.π₁ f p₁ p₂).Final := sorry

instance : (Index.π₂ f p₁ p₂).Final := sorry

section

variable [IsCardinalAccessibleCategory C₁ κ] [IsCardinalAccessibleCategory C₂ κ]
[IsCardinalAccessibleCategory D κ]
[F₁.IsCardinalAccessible κ] [F₂.IsCardinalAccessible κ]

def isColimitCocone : IsColimit (cocone f p₁ p₂) := sorry
def isColimitCocone : IsColimit (cocone f p₁ p₂) := by
sorry

noncomputable def cardinalFilteredPresentation :
CardinalFilteredPresentation (Comma.mk _ _ f) κ :=
Expand Down

0 comments on commit 8b9474e

Please sign in to comment.