Zulip Chat Archive
Stream: Is there code for X?
Topic: Schemes isomorphic to affine schemes are affine
Michał Mrugała (Mar 17 2025 at 14:36):
I'm very surprised that the following examples are not closed by exact?
. They shouldn't be difficult to prove using mem_Spec_essImage
, but am I missing something obvious here? Should these be added to Mathlib?
import Mathlib.AlgebraicGeometry.AffineScheme
open AlgebraicGeometry
variable {X : Scheme}
example {Y : Scheme} [IsAffine Y] (h : X ≅ Y) : IsAffine X := sorry --by exact?
example {R : CommRingCat} (h : X ≅ Spec R) : IsAffine X := sorry --by exact?
Markus Himmel (Mar 17 2025 at 14:43):
docs#AlgebraicGeometry.isAffine_of_isIso exists, it's a bit sad (but not surprising) that exact?
cannot find it.
Michał Mrugała (Mar 17 2025 at 14:52):
Thanks, this is exactly what I needed. Do you think it's worth PRing the "morphism"-free version?
Last updated: May 02 2025 at 03:31 UTC