Documentation

Mathlib.AlgebraicGeometry.Morphisms.QuasiCompact

Quasi-compact morphisms #

A morphism of schemes is quasi-compact if the preimages of quasi-compact open sets are quasi-compact.

It suffices to check that preimages of affine open sets are compact (quasiCompact_iff_forall_affine).

A morphism is "quasi-compact" if the underlying map of topological spaces is, i.e. if the preimages of quasi-compact open sets are quasi-compact.

Instances
    theorem AlgebraicGeometry.isCompact_basicOpen (X : Scheme) {U : X.Opens} (hU : IsCompact U) (f : (X.presheaf.obj (Opposite.op U))) :
    theorem AlgebraicGeometry.compact_open_induction_on {X : Scheme} {P : X.OpensProp} (S : X.Opens) (hS : IsCompact S.carrier) (h₁ : P ) (h₂ : ∀ (S : X.Opens), IsCompact S.carrier∀ (U : X.affineOpens), P SP (S U)) :
    P S

    If x : Γ(X, U) is zero on D(f) for some f : Γ(X, U), and U is quasi-compact, then f ^ n * x = 0 for some n.

    A section over a compact open of a scheme is nilpotent if and only if its associated basic open is empty.

    A global section of a quasi-compact scheme is nilpotent if and only if its associated basic open is empty.

    The zero locus of a set of sections over a compact open of a scheme is X if and only if s is contained in the nilradical of Γ(X, U).

    The zero locus of a set of sections over a compact open of a scheme is X if and only if s is contained in the nilradical of Γ(X, U).