Skip to content

Commit 3830f92

Browse files
committed
chore: remove use of erw in Geometry.RingedSpace.OpenImmersion (#31856)
1 parent 50f57fe commit 3830f92

File tree

1 file changed

+2
-1
lines changed

1 file changed

+2
-1
lines changed

Mathlib/Geometry/RingedSpace/OpenImmersion.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -491,7 +491,8 @@ def lift (H : Set.range g.base ⊆ Set.range f.base) : Y ⟶ X :=
491491

492492
@[simp, reassoc]
493493
theorem lift_fac (H : Set.range g.base ⊆ Set.range f.base) : lift f g H ≫ f = g := by
494-
erw [Category.assoc]; rw [IsIso.inv_comp_eq]; exact pullback.condition
494+
simp [AlgebraicGeometry.PresheafedSpace.IsOpenImmersion.lift,
495+
CategoryTheory.Limits.pullback.condition]
495496

496497
theorem lift_uniq (H : Set.range g.base ⊆ Set.range f.base) (l : Y ⟶ X) (hl : l ≫ f = g) :
497498
l = lift f g H := by rw [← cancel_mono f, hl, lift_fac]

0 commit comments

Comments
 (0)