Skip to content

Commit aa5b6a4

Browse files
committed
feat(AlgebraicGeometry): define affine n-space (#18837)
Co-authored-by: Andrew Yang <36414270+erdOne@users.noreply.github.com>
1 parent 4621579 commit aa5b6a4

File tree

3 files changed

+391
-0
lines changed

3 files changed

+391
-0
lines changed

Mathlib.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -907,6 +907,7 @@ import Mathlib.Algebra.Tropical.BigOperators
907907
import Mathlib.Algebra.Tropical.Lattice
908908
import Mathlib.Algebra.Vertex.HVertexOperator
909909
import Mathlib.AlgebraicGeometry.AffineScheme
910+
import Mathlib.AlgebraicGeometry.AffineSpace
910911
import Mathlib.AlgebraicGeometry.Cover.MorphismProperty
911912
import Mathlib.AlgebraicGeometry.Cover.Open
912913
import Mathlib.AlgebraicGeometry.EllipticCurve.Affine

Mathlib/AlgebraicGeometry/AffineScheme.lean

Lines changed: 4 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -134,6 +134,10 @@ theorem Scheme.isoSpec_Spec (R : CommRingCat.{u}) :
134134
(Spec R).isoSpec.inv = Spec.map (Scheme.ΓSpecIso R).inv :=
135135
congr($(isoSpec_Spec R).inv)
136136

137+
lemma ext_of_isAffine {X Y : Scheme} [IsAffine Y] {f g : X ⟶ Y} (e : f.app ⊤ = g.app ⊤) :
138+
f = g := by
139+
rw [← cancel_mono Y.toSpecΓ, Scheme.toSpecΓ_naturality, Scheme.toSpecΓ_naturality, e]
140+
137141
namespace AffineScheme
138142

139143
/-- The `Spec` functor into the category of affine schemes. -/

0 commit comments

Comments
 (0)