Skip to content

Commit a105877

Browse files
committed
fix
1 parent 0e3384c commit a105877

File tree

2 files changed

+6
-10
lines changed

2 files changed

+6
-10
lines changed

Mathlib/AlgebraicGeometry/Morphisms/ClosedImmersion.lean

+1-5
Original file line numberDiff line numberDiff line change
@@ -47,10 +47,6 @@ lemma closedEmbedding {X Y : Scheme} (f : X ⟶ Y)
4747
[IsClosedImmersion f] : ClosedEmbedding f.1.base :=
4848
IsClosedImmersion.base_closed
4949

50-
lemma surjective_stalkMap {X Y : Scheme} (f : X ⟶ Y)
51-
[IsClosedImmersion f] (x : X) : Function.Surjective (f.stalkMap x) :=
52-
IsClosedImmersion.surj_on_stalks x
53-
5450
lemma eq_inf : @IsClosedImmersion = (topologically ClosedEmbedding) ⊓
5551
stalkwise (fun f ↦ Function.Surjective f) := by
5652
ext X Y f
@@ -132,7 +128,7 @@ theorem of_comp {X Y Z : Scheme} (f : X ⟶ Y) (g : Y ⟶ Z) [IsClosedImmersion
132128
← Set.image_comp]
133129
exact ClosedEmbedding.isClosedMap h _ hZ
134130
surj_on_stalks x := by
135-
have h := surjective_stalkMap (f ≫ g) x
131+
have h := (f ≫ g).stalkMap_surjective x
136132
simp_rw [Scheme.comp_val, Scheme.stalkMap_comp] at h
137133
exact Function.Surjective.of_comp h
138134

Mathlib/AlgebraicGeometry/Morphisms/Preimmersion.lean

+5-5
Original file line numberDiff line numberDiff line change
@@ -34,13 +34,13 @@ topological spaces is an embedding and the induced morphisms of stalks are all s
3434
@[mk_iff]
3535
class IsPreimmersion {X Y : Scheme} (f : X ⟶ Y) : Prop where
3636
base_embedding : Embedding f.1.base
37-
surj_on_stalks : ∀ x, Function.Surjective (PresheafedSpace.stalkMap f.1 x)
37+
surj_on_stalks : ∀ x, Function.Surjective (f.stalkMap x)
3838

3939
lemma Scheme.Hom.embedding {X Y : Scheme} (f : Hom X Y) [IsPreimmersion f] : Embedding f.1.base :=
4040
IsPreimmersion.base_embedding
4141

4242
lemma Scheme.Hom.stalkMap_surjective {X Y : Scheme} (f : Hom X Y) [IsPreimmersion f] (x) :
43-
Function.Surjective (PresheafedSpace.stalkMap f.1 x) :=
43+
Function.Surjective (f.stalkMap x) :=
4444
IsPreimmersion.surj_on_stalks x
4545

4646
lemma isPreimmersion_eq_inf :
@@ -51,7 +51,7 @@ lemma isPreimmersion_eq_inf :
5151

5252
/-- Being surjective on stalks is local at the target. -/
5353
instance isSurjectiveOnStalks_isLocalAtTarget : IsLocalAtTarget
54-
(stalkwise (fun f ↦ Function.Surjective f)) :=
54+
(stalkwise (Function.Surjective ·)) :=
5555
stalkwiseIsLocalAtTarget_of_respectsIso surjective_respectsIso
5656

5757
namespace IsPreimmersion
@@ -67,7 +67,7 @@ instance : MorphismProperty.IsMultiplicative @IsPreimmersion where
6767
id_mem _ := inferInstance
6868
comp_mem {X Y Z} f g hf hg := by
6969
refine ⟨hg.base_embedding.comp hf.base_embedding, fun x ↦ ?_⟩
70-
erw [PresheafedSpace.stalkMap.comp]
70+
rw [Scheme.stalkMap_comp]
7171
exact (hf.surj_on_stalks x).comp (hg.surj_on_stalks (f.1.1 x))
7272

7373
instance comp {X Y Z : Scheme} (f : X ⟶ Y) (g : Y ⟶ Z) [IsPreimmersion f]
@@ -88,7 +88,7 @@ theorem of_comp {X Y Z : Scheme} (f : X ⟶ Y) (g : Y ⟶ Z) [IsPreimmersion g]
8888
rwa [← g.embedding.of_comp_iff]
8989
surj_on_stalks x := by
9090
have h := (f ≫ g).stalkMap_surjective x
91-
erw [Scheme.comp_val, PresheafedSpace.stalkMap.comp] at h
91+
rw [Scheme.stalkMap_comp] at h
9292
exact Function.Surjective.of_comp h
9393

9494
theorem comp_iff {X Y Z : Scheme} (f : X ⟶ Y) (g : Y ⟶ Z) [IsPreimmersion g] :

0 commit comments

Comments
 (0)