Skip to content

Commit 2fc3307

Browse files
committed
fix
1 parent c08f944 commit 2fc3307

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

Mathlib/AlgebraicGeometry/Restrict.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -117,7 +117,7 @@ def stalkIso {X : Scheme.{u}} (U : X.Opens) (x : U) :
117117

118118
@[reassoc (attr := simp)]
119119
lemma germ_stalkIso_hom {X : Scheme.{u}} (U : X.Opens)
120-
{V : TopologicalSpace.Opens U} (x : V) :
120+
{V : TopologicalSpace.Opens U} (x : V) :
121121
U.toScheme.presheaf.germ x ≫ (U.stalkIso x.1).hom =
122122
X.presheaf.germ ⟨x.1.1, show x.1.1 ∈ U.ι ''ᵁ V from ⟨x.1, x.2, rfl⟩⟩ :=
123123
PresheafedSpace.restrictStalkIso_hom_eq_germ _ _ _ _ _

0 commit comments

Comments
 (0)