@@ -371,6 +371,42 @@ lemma stalkMap_inv_hom {X Y : LocallyRingedSpace.{u}} (e : X ≅ Y) (x : X) :
371
371
rw [← stalkMap_comp, LocallyRingedSpace.stalkMap_congr_hom (e.hom ≫ e.inv) (𝟙 _) (by simp)]
372
372
simp
373
373
374
+ @[reassoc, elementwise]
375
+ lemma stalkMap_germ {X Y : LocallyRingedSpace.{u}} (f : X ⟶ Y) (U : Opens Y)
376
+ (x : (Opens.map f.val.base).obj U) :
377
+ Y.presheaf.germ ⟨f.val.base x.val, x.property⟩ ≫ f.stalkMap x.val =
378
+ f.val.c.app (op U) ≫ X.presheaf.germ x :=
379
+ PresheafedSpace.stalkMap_germ f.val U x
380
+
381
+ @[reassoc (attr := simp), elementwise (attr := simp)]
382
+ lemma stalkMap_germ' {X Y : LocallyRingedSpace.{u}} (f : X ⟶ Y) (U : Opens Y) (x : X)
383
+ (hx : f.val.base x ∈ U) :
384
+ Y.presheaf.germ ⟨f.val.base x, hx⟩ ≫ f.stalkMap x =
385
+ f.val.c.app (op U) ≫ X.presheaf.germ (U := (Opens.map f.val.base).obj U) ⟨x, hx⟩ :=
386
+ PresheafedSpace.stalkMap_germ' f.val U x hx
387
+
388
+ variable {U : TopCat} (X : LocallyRingedSpace.{u}) {f : U ⟶ X.toTopCat} (h : OpenEmbedding f)
389
+ (V : Opens U) (x : U) (hx : x ∈ V)
390
+
391
+ @[elementwise, reassoc]
392
+ lemma restrictStalkIso_hom_eq_germ :
393
+ (X.restrict h).presheaf.germ ⟨x, hx⟩ ≫ (X.restrictStalkIso h x).hom =
394
+ X.presheaf.germ ⟨f x, show f x ∈ h.isOpenMap.functor.obj V from ⟨x, hx, rfl⟩⟩ :=
395
+ PresheafedSpace.restrictStalkIso_hom_eq_germ X.toPresheafedSpace h V x hx
396
+
397
+ @[simp, elementwise, reassoc]
398
+ lemma restrictStalkIso_inv_eq_germ :
399
+ X.presheaf.germ ⟨f x, show f x ∈ h.isOpenMap.functor.obj V from ⟨x, hx, rfl⟩⟩ ≫
400
+ (X.restrictStalkIso h x).inv = (X.restrict h).presheaf.germ ⟨x, hx⟩ :=
401
+ PresheafedSpace.restrictStalkIso_inv_eq_germ X.toPresheafedSpace h V x hx
402
+
403
+ lemma restrictStalkIso_inv_eq_ofRestrict :
404
+ (X.restrictStalkIso h x).inv = (X.ofRestrict h).stalkMap x :=
405
+ PresheafedSpace.restrictStalkIso_inv_eq_ofRestrict X.toPresheafedSpace h x
406
+
407
+ instance ofRestrict_stalkMap_isIso : IsIso ((X.ofRestrict h).stalkMap x) :=
408
+ PresheafedSpace.ofRestrict_stalkMap_isIso X.toPresheafedSpace h x
409
+
374
410
end Stalks
375
411
376
412
end LocallyRingedSpace
0 commit comments