Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 996783c

Browse files
feat(topology/sheaves/stalks): Generalize from Type to algebraic categories (#9357)
Previously, basic lemmas about stalks like `germ_exist` and `section_ext` were only available for `Type`-valued (pre)sheaves. This PR generalizes these to (pre)sheaves valued in any concrete category where the forgetful functor preserves filtered colimits, which includes most algebraic categories like `Group` and `CommRing`. For the statements about stalks maps, we additionally assume that the forgetful functor reflects isomorphisms and preserves limits.
1 parent 865ad47 commit 996783c

File tree

2 files changed

+220
-195
lines changed

2 files changed

+220
-195
lines changed

src/topology/sheaves/sheafify.lean

Lines changed: 4 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -70,7 +70,7 @@ sending each section to its germs.
7070
-/
7171
def to_sheafify : F ⟶ F.sheafify.presheaf :=
7272
{ app := λ U f, ⟨λ x, F.germ x f, prelocal_predicate.sheafify_of ⟨f, λ x, rfl⟩⟩,
73-
naturality' := λ U U' f, by { ext x ⟨u, m⟩, apply germ_res_apply', }, }
73+
naturality' := λ U U' f, by { ext x ⟨u, m⟩, exact germ_res_apply F f.unop ⟨u, m⟩ x } }
7474

7575
/--
7676
The natural morphism from the stalk of the sheafification to the original stalk.
@@ -101,6 +101,7 @@ begin
101101
have wVx := wV ⟨x, mV⟩,
102102
dsimp at wVx, erw wVx at e, clear wVx,
103103
rcases F.germ_eq x mU mV gU gV e with ⟨W, mW, iU', iV', e'⟩,
104+
dsimp at e',
104105
use ⟨W ⊓ (U' ⊓ V'), ⟨mW, mU, mV⟩⟩,
105106
refine ⟨_, _, _⟩,
106107
{ change W ⊓ (U' ⊓ V') ⟶ U.val,
@@ -113,8 +114,8 @@ begin
113114
dsimp at wU,
114115
specialize wV ⟨w.1, w.2.2.2⟩,
115116
dsimp at wV,
116-
erw [wU, ←F.germ_res_apply iU' ⟨w, w.2.1 gU, e', F.germ_res_apply, ←wV],
117-
refl, },
117+
erw [wU, ←F.germ_res iU' ⟨w, w.2.1, wV, ←F.germ_res iV' ⟨w, w.2.1,
118+
category_theory.types_comp_apply, category_theory.types_comp_apply, e'] },
118119
end
119120

120121
/--

0 commit comments

Comments
 (0)