Quasi-finite morphisms #
We say that a morphism f : X ⟶ Y is locally quasi finite if Γ(Y, U) ⟶ Γ(X, V) is
quasi-finite (in the mathlib sense) for every pair of affine opens that f maps one into the other.
This is equivalent to all the fibers f⁻¹(x) having an open cover of κ(x)-finite schemes.
Note that this does not require f to be quasi-compact nor locally of finite type.
We prove that this is stable under composition and base change, and is right cancellative.
TODO (@erdOne): #
- If
fis quasi-compact, thenfis locally quasi-finite iff all the fibersf⁻¹(x)areκ(x)-finite. - If
fis locally of finite type, thenfis locally quasi-finite ifffhas discrete fibers. - If
fis of finite type, thenfis locally quasi-finite ifffhas finite fibers.
We say that a morphism f : X ⟶ Y is locally quasi finite if Γ(Y, U) ⟶ Γ(X, V) is
quasi-finite (in the mathlib sense) for every pair of affine opens that f maps one into the other.
This is equivalent to all the fibers f⁻¹(x) having an open cover of κ(x)-finite schemes.
Note that this does not require f to be quasi-compact nor locally of finite type.
TODO (@erdOne): prove the following
If one assumes quasi-compact, this is equivalent to all the fibers f⁻¹(x) being κ(x)-finite.
If one assumes locally of finite type, this is equivalent to f having discrete fibers.
If one assumes finite type, this is equivalent to f having finite fibers.
- quasiFinite_appLE {U : Y.Opens} : IsAffineOpen U → ∀ {V : X.Opens}, IsAffineOpen V → ∀ (e : V ≤ (TopologicalSpace.Opens.map f.base).obj U), (CommRingCat.Hom.hom (Scheme.Hom.appLE f U V e)).QuasiFinite