Skip to content

Commit

Permalink
fix errors
Browse files Browse the repository at this point in the history
  • Loading branch information
dagurtomas committed Aug 26, 2024
1 parent a85395e commit a042432
Showing 1 changed file with 1 addition and 0 deletions.
1 change: 1 addition & 0 deletions LeanCondensed/LightCondensed/SequentialLimit.lean
Original file line number Diff line number Diff line change
Expand Up @@ -76,6 +76,7 @@ variable (R : Type*) [Ring R]
variable {F : ℕᵒᵖ ⥤ LightCondMod R} {c : Cone F} (hc : IsLimit c)
(hF : ∀ n, Epi (F.map (homOfLE (Nat.le_succ n)).op))

include hc hF in
lemma epi_limit_of_epi : Epi (c.π.app ⟨0⟩) := by
rw [LightCondMod.epi_iff_locallySurjective_on_lightProfinite]
intro S g
Expand Down

0 comments on commit a042432

Please sign in to comment.