We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
erw
Geometry.RingedSpace.OpenImmersion
1 parent 50f57fe commit 3830f92Copy full SHA for 3830f92
Mathlib/Geometry/RingedSpace/OpenImmersion.lean
@@ -491,7 +491,8 @@ def lift (H : Set.range g.base ⊆ Set.range f.base) : Y ⟶ X :=
491
492
@[simp, reassoc]
493
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
+ simp [AlgebraicGeometry.PresheafedSpace.IsOpenImmersion.lift,
495
+ CategoryTheory.Limits.pullback.condition]
496
497
theorem lift_uniq (H : Set.range g.base ⊆ Set.range f.base) (l : Y ⟶ X) (hl : l ≫ f = g) :
498
l = lift f g H := by rw [← cancel_mono f, hl, lift_fac]
0 commit comments