Skip to content

Commit

Permalink
Fix
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Feb 22, 2025
1 parent fd0ba47 commit 2c8cb11
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Analysis/SpecialFunctions/PolarCoord.lean
Original file line number Diff line number Diff line change
Expand Up @@ -78,7 +78,7 @@ def polarCoord : PartialHomeomorph (ℝ × ℝ) (ℝ × ℝ) where
(isOpen_ne_fun continuous_snd continuous_const)
continuousOn_invFun := by fun_prop
continuousOn_toFun := by
refine .prod_mk (by fun_prop) ?_
refine .prod (by fun_prop) ?_
have A : MapsTo Complex.equivRealProd.symm ({q : ℝ × ℝ | 0 < q.1} ∪ {q : ℝ × ℝ | q.20})
Complex.slitPlane := by
rintro ⟨x, y⟩ hxy; simpa only using hxy
Expand Down

0 comments on commit 2c8cb11

Please sign in to comment.