-
Notifications
You must be signed in to change notification settings - Fork 384
New issue
Have a question about this project? Sign up for a free GitHub account to open an issue and contact its maintainers and the community.
By clicking “Sign up for GitHub”, you agree to our terms of service and privacy statement. We’ll occasionally send you account related emails.
Already on GitHub? Sign in to your account
[Merged by Bors] - feat(AlgebraicGeometry/GammaSpecAdjunction): a missing lemma #13412
Conversation
This is a fun error: Error: ././././Mathlib/AlgebraicGeometry/GammaSpecAdjunction.lean:371:9: error: AlgebraicGeometry.ΓSpec.locallyRingedSpaceAdjunction_homEquiv_apply.{u_1} Left-hand side simplifies from
(AlgebraicGeometry.ΓSpec.locallyRingedSpaceAdjunction.homEquiv X R) f
to
(AlgebraicGeometry.ΓSpec.locallyRingedSpaceAdjunction.homEquiv X R) f They look the same to me. |
Looking at the lemmas used, I think some implicit types involved were dsimped. import Mathlib.Logic.Equiv.Defs
def A := Unit
@[simp] def B := A
def e : B ≃ Unit := Equiv.refl _
@[simp] lemma e_apply (x) : e x = x := rfl
example (x) : e x = x := by simp -- fails because `B` gets rewritten to `A` first.
#lint only simpNF |
Maybe either raise its priority or don't tag it as simp. |
Raising priority to high doesn't seem to be working, so I deleted the simp attribute |
Co-authored-by: github-actions[bot] <41898282+github-actions[bot]@users.noreply.github.com>
…leanprover-community/mathlib4 into zjj/GammaSpecAdj_missing_lemmas
Co-authored-by: Junyan Xu <[email protected]>
Co-authored-by: Andrew Yang <[email protected]>
…leanprover-community/mathlib4 into zjj/GammaSpecAdj_missing_lemmas
PR summaryImport changesNo significant changes to the import graph
|
Thanks! bors merge |
Added the following lemma: Let $X$ be a locally ringed space, $R$ a ring and $U \subseteq \mathrm{Spec} R$ an open set. Then for any $f : R \to \Gamma(\mathcal O_X, X)$, if we denote $F$ as the corresponding morphism $X \to \mathrm{Spec} R$ under the gamma spec adjunction we have that the composition $res^{\mathrm{X}}\_{F^{-1}U} \circ f$ is equal to the composition $(R \to \mathcal{O}_{\mathrm{Spec} R}(U)\circ F(U)$ ```lean lemma toOpen_comp_locallyRingedSpaceAdjunction_homEquiv_app {X : LocallyRingedSpace} {R : Type u} [CommRing R] (f : LocallyRingedSpace.Γ.rightOp.obj X ⟶ op (CommRingCat.of R)) (U) : StructureSheaf.toOpen R U.unop ≫ (locallyRingedSpaceAdjunction.homEquiv X (op <| CommRingCat.of R) f).1.c.app U = f.unop ≫ X.presheaf.map (homOfLE le_top).op := by ``` found usefuly by Andrew during #12371 Co-authored-by: Andrew Yang <[email protected]>
Pull request successfully merged into master. Build succeeded: |
Added the following lemma: Let $X$ be a locally ringed space, $R$ a ring and $U \subseteq \mathrm{Spec} R$ an open set. Then for any $f : R \to \Gamma(\mathcal O_X, X)$, if we denote $F$ as the corresponding morphism $X \to \mathrm{Spec} R$ under the gamma spec adjunction we have that the composition $res^{\mathrm{X}}\_{F^{-1}U} \circ f$ is equal to the composition $(R \to \mathcal{O}_{\mathrm{Spec} R}(U)\circ F(U)$ ```lean lemma toOpen_comp_locallyRingedSpaceAdjunction_homEquiv_app {X : LocallyRingedSpace} {R : Type u} [CommRing R] (f : LocallyRingedSpace.Γ.rightOp.obj X ⟶ op (CommRingCat.of R)) (U) : StructureSheaf.toOpen R U.unop ≫ (locallyRingedSpaceAdjunction.homEquiv X (op <| CommRingCat.of R) f).1.c.app U = f.unop ≫ X.presheaf.map (homOfLE le_top).op := by ``` found usefuly by Andrew during #12371 Co-authored-by: Andrew Yang <[email protected]>
Added the following lemma:
Let$X$ be a locally ringed space, $R$ a ring and $U \subseteq \mathrm{Spec} R$ an open set.$f : R \to \Gamma(\mathcal O_X, X)$ , if we denote $F$ as the corresponding morphism $X \to \mathrm{Spec} R$ under the gamma spec adjunction we have that$res^{\mathrm{X}}_{F^{-1}U} \circ f$ is equal to the composition $(R \to \mathcal{O}_{\mathrm{Spec} R}(U)\circ F(U)$
Then for any
the composition
found usefuly by Andrew during #12371
Co-authored-by: Andrew Yang [email protected]