@@ -34,13 +34,13 @@ topological spaces is an embedding and the induced morphisms of stalks are all s
34
34
@[mk_iff]
35
35
class IsPreimmersion {X Y : Scheme} (f : X ⟶ Y) : Prop where
36
36
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)
38
38
39
39
lemma Scheme.Hom.embedding {X Y : Scheme} (f : Hom X Y) [IsPreimmersion f] : Embedding f.1 .base :=
40
40
IsPreimmersion.base_embedding
41
41
42
42
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) :=
44
44
IsPreimmersion.surj_on_stalks x
45
45
46
46
lemma isPreimmersion_eq_inf :
@@ -51,7 +51,7 @@ lemma isPreimmersion_eq_inf :
51
51
52
52
/-- Being surjective on stalks is local at the target. -/
53
53
instance isSurjectiveOnStalks_isLocalAtTarget : IsLocalAtTarget
54
- (stalkwise (fun f ↦ Function.Surjective f )) :=
54
+ (stalkwise (Function.Surjective · )) :=
55
55
stalkwiseIsLocalAtTarget_of_respectsIso surjective_respectsIso
56
56
57
57
namespace IsPreimmersion
@@ -67,7 +67,7 @@ instance : MorphismProperty.IsMultiplicative @IsPreimmersion where
67
67
id_mem _ := inferInstance
68
68
comp_mem {X Y Z} f g hf hg := by
69
69
refine ⟨hg.base_embedding.comp hf.base_embedding, fun x ↦ ?_⟩
70
- erw [PresheafedSpace.stalkMap.comp ]
70
+ rw [Scheme.stalkMap_comp ]
71
71
exact (hf.surj_on_stalks x).comp (hg.surj_on_stalks (f.1 .1 x))
72
72
73
73
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]
88
88
rwa [← g.embedding.of_comp_iff]
89
89
surj_on_stalks x := by
90
90
have h := (f ≫ g).stalkMap_surjective x
91
- erw [Scheme.comp_val, PresheafedSpace.stalkMap.comp ] at h
91
+ rw [Scheme.stalkMap_comp ] at h
92
92
exact Function.Surjective.of_comp h
93
93
94
94
theorem comp_iff {X Y Z : Scheme} (f : X ⟶ Y) (g : Y ⟶ Z) [IsPreimmersion g] :
0 commit comments