Skip to content

Commit

Permalink
fix(*): arsinh and complex.basic had module docs at the wrong position (
Browse files Browse the repository at this point in the history
#6230)

This is fixed and the module doc for `complex.basic` is expanded slightly.
  • Loading branch information
Julian-Kuelshammer committed Feb 14, 2021
1 parent c54a8d0 commit b9af22d
Show file tree
Hide file tree
Showing 2 changed files with 6 additions and 4 deletions.
2 changes: 1 addition & 1 deletion src/analysis/special_functions/arsinh.lean
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: James Arthur, Chris Hughes, Shing Tak Lam
-/
import analysis.special_functions.trigonometric
noncomputable theory

/-!
# Inverse of the sinh function
Expand All @@ -23,6 +22,7 @@ inverse, arsinh.
arsinh, arcsinh, argsinh, asinh, sinh injective, sinh bijective, sinh surjective
-/
noncomputable theory

namespace real

Expand Down
8 changes: 5 additions & 3 deletions src/data/complex/basic.lean
Expand Up @@ -5,14 +5,16 @@ Authors: Kevin Buzzard, Mario Carneiro
-/
import data.real.sqrt

open_locale big_operators

/-!
# The complex numbers
The complex numbers are modelled as ℝ^2 in the obvious way.
The complex numbers are modelled as ℝ^2 in the obvious way and it is shown that they form a field
of characteristic zero. The result that the complex numbers are algebraically closed, see
`field_theory.algebraic_closure`.
-/

open_locale big_operators

/-! ### Definition and basic arithmmetic -/

/-- Complex numbers consist of two `real`s: a real part `re` and an imaginary part `im`. -/
Expand Down

0 comments on commit b9af22d

Please sign in to comment.