Skip to content

Commit

Permalink
style: use exact instead of refine'.
Browse files Browse the repository at this point in the history
  • Loading branch information
grunweg committed Jan 25, 2024
1 parent a4d52e2 commit 7243e44
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion SphereEversion/Loops/Surrounding.lean
Original file line number Diff line number Diff line change
Expand Up @@ -998,7 +998,7 @@ theorem exists_surrounding_loops (hK : IsClosed K) (hΩ_op : IsOpen Ω) (hg :
(surroundingFamilyIn_iff_germ.mpr ⟨hγ₂, h'γ₂⟩) with
⟨U, U_in, γ, H, H''⟩
cases' surroundingFamilyIn_iff_germ.mp H with H H'
refine' ⟨γ, H, mem_of_superset U_in H', Eventually.union_nhdsSet.mpr H''⟩
exact ⟨γ, H, mem_of_superset U_in H', Eventually.union_nhdsSet.mpr H''⟩

-- #lint
-- #print axioms satisfied_or_refund
Expand Down

0 comments on commit 7243e44

Please sign in to comment.