Skip to content

Commit

Permalink
feat (analysis/special_functions): limit formula and reflection formu…
Browse files Browse the repository at this point in the history
…la for Gamma (#18404)

This adds Euler's limit formula and the reflection formula for the Gamma function. As a consequence we get that Gamma
does not vanish on the complex plane (except at non-positive integers, where it is undefined, and we have arbitrarily chosen it to be 0).
  • Loading branch information
loefflerd committed Feb 15, 2023
1 parent 1ead223 commit 372edc3
Show file tree
Hide file tree
Showing 4 changed files with 413 additions and 48 deletions.
5 changes: 5 additions & 0 deletions src/analysis/normed/field/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -487,6 +487,11 @@ begin
simp,
end

/-- A normed division ring is a topological division ring. -/
@[priority 100] -- see Note [lower instance priority]
instance normed_division_ring.to_topological_division_ring : topological_division_ring α :=
{ }

lemma norm_map_one_of_pow_eq_one [monoid β] (φ : β →* α) {x : β} {k : ℕ+}
(h : x ^ (k : ℕ) = 1) :
‖φ x‖ = 1 :=
Expand Down
Loading

0 comments on commit 372edc3

Please sign in to comment.