Skip to content

Commit

Permalink
chore(AlgebraicGeometry/Gluing): fix soon-to-be-broken proof (#11838)
Browse files Browse the repository at this point in the history
This proof had two `change`s added during porting, and these produce a massive timeout after the changes in leanprover/lean4#3807.

This PR replace the `change` with the appropriate `erw`, and is now fast before and after the change.

Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
  • Loading branch information
2 people authored and callesonne committed Apr 22, 2024
1 parent 453aedd commit f5d321c
Showing 1 changed file with 2 additions and 6 deletions.
8 changes: 2 additions & 6 deletions Mathlib/AlgebraicGeometry/Gluing.lean
Original file line number Diff line number Diff line change
Expand Up @@ -379,12 +379,8 @@ theorem fromGlued_injective : Function.Injective 𝒰.fromGlued.1.base := by
right
use e.hom ⟨⟨x, y⟩, h⟩
constructor
-- Porting note: in the two subproofs below, added the `change` lines
· change (e.hom ≫ _) ⟨(x, y), h⟩ = x
erw [IsLimit.conePointUniqueUpToIso_hom_comp _ _ WalkingCospan.left]; rfl
· change (e.hom ≫ ((gluedCover 𝒰).toGlueData.t i j ≫
(gluedCover 𝒰).toGlueData.f j i).val.base) ⟨(x, y), h⟩ = y
erw [pullbackSymmetry_hom_comp_fst,
· erw [← comp_apply e.hom, IsLimit.conePointUniqueUpToIso_hom_comp _ _ WalkingCospan.left]; rfl
· erw [← comp_apply e.hom, pullbackSymmetry_hom_comp_fst,
IsLimit.conePointUniqueUpToIso_hom_comp _ _ WalkingCospan.right]
rfl
#align algebraic_geometry.Scheme.open_cover.from_glued_injective AlgebraicGeometry.Scheme.OpenCover.fromGlued_injective
Expand Down

0 comments on commit f5d321c

Please sign in to comment.