Skip to content

Commit

Permalink
restore a proof
Browse files Browse the repository at this point in the history
  • Loading branch information
Scott Morrison authored and semorrison committed Jun 8, 2023
1 parent b6e86a2 commit ae8d859
Showing 1 changed file with 1 addition and 0 deletions.
1 change: 1 addition & 0 deletions Mathlib/CategoryTheory/Sites/Plus.lean
Original file line number Diff line number Diff line change
Expand Up @@ -57,6 +57,7 @@ def diagramPullback {X Y : C} (f : X ⟶ Y) : J.diagram P Y ⟶ (J.pullback f).o
app S :=
Multiequalizer.lift _ _ (fun I => Multiequalizer.ι (S.unop.index P) I.base) fun I =>
Multiequalizer.condition (S.unop.index P) I.base
naturality S T f := Multiequalizer.hom_ext _ _ _ (fun I => by dsimp ; simp ; rfl)
#align category_theory.grothendieck_topology.diagram_pullback CategoryTheory.GrothendieckTopology.diagramPullback

/-- A natural transformation `P ⟶ Q` induces a natural transformation
Expand Down

0 comments on commit ae8d859

Please sign in to comment.