Documentation

Mathlib.Analysis.SpecialFunctions.Trigonometric.Inverse

Inverse trigonometric functions. #

See also Analysis.SpecialFunctions.Trigonometric.Arctan for the inverse tan function. (This is delayed as it is easier to set up after developing complex trigonometric functions.)

Basic inequalities on trigonometric functions.

noncomputable def Real.arcsin :

Inverse of the sin function, returns values in the range -π / 2 ≤ arcsin x ≤ π / 2. It defaults to -π / 2 on (-∞, -1) and to π / 2 to (1, ∞).

Equations
Instances For
    theorem Real.arcsin_mem_Icc (x : ) :
    x.arcsin Set.Icc (-(Real.pi / 2)) (Real.pi / 2)
    theorem Real.arcsin_le_pi_div_two (x : ) :
    x.arcsin Real.pi / 2
    theorem Real.arcsin_projIcc (x : ) :
    ((Set.projIcc (-1) 1 x)).arcsin = x.arcsin
    theorem Real.sin_arcsin' {x : } (hx : x Set.Icc (-1) 1) :
    x.arcsin.sin = x
    theorem Real.sin_arcsin {x : } (hx₁ : -1 x) (hx₂ : x 1) :
    x.arcsin.sin = x
    theorem Real.arcsin_sin' {x : } (hx : x Set.Icc (-(Real.pi / 2)) (Real.pi / 2)) :
    x.sin.arcsin = x
    theorem Real.arcsin_sin {x : } (hx₁ : -(Real.pi / 2) x) (hx₂ : x Real.pi / 2) :
    x.sin.arcsin = x
    theorem Real.arcsin_inj {x : } {y : } (hx₁ : -1 x) (hx₂ : x 1) (hy₁ : -1 y) (hy₂ : y 1) :
    x.arcsin = y.arcsin x = y
    theorem Real.arcsin_eq_of_sin_eq {x : } {y : } (h₁ : x.sin = y) (h₂ : x Set.Icc (-(Real.pi / 2)) (Real.pi / 2)) :
    y.arcsin = x
    @[simp]
    theorem Real.arcsin_of_one_le {x : } (hx : 1 x) :
    x.arcsin = Real.pi / 2
    theorem Real.arcsin_neg_one :
    (-1).arcsin = -(Real.pi / 2)
    theorem Real.arcsin_of_le_neg_one {x : } (hx : x -1) :
    x.arcsin = -(Real.pi / 2)
    @[simp]
    theorem Real.arcsin_neg (x : ) :
    (-x).arcsin = -x.arcsin
    theorem Real.arcsin_le_iff_le_sin {x : } {y : } (hx : x Set.Icc (-1) 1) (hy : y Set.Icc (-(Real.pi / 2)) (Real.pi / 2)) :
    x.arcsin y x y.sin
    theorem Real.arcsin_le_iff_le_sin' {x : } {y : } (hy : y Set.Ico (-(Real.pi / 2)) (Real.pi / 2)) :
    x.arcsin y x y.sin
    theorem Real.le_arcsin_iff_sin_le {x : } {y : } (hx : x Set.Icc (-(Real.pi / 2)) (Real.pi / 2)) (hy : y Set.Icc (-1) 1) :
    x y.arcsin x.sin y
    theorem Real.le_arcsin_iff_sin_le' {x : } {y : } (hx : x Set.Ioc (-(Real.pi / 2)) (Real.pi / 2)) :
    x y.arcsin x.sin y
    theorem Real.arcsin_lt_iff_lt_sin {x : } {y : } (hx : x Set.Icc (-1) 1) (hy : y Set.Icc (-(Real.pi / 2)) (Real.pi / 2)) :
    x.arcsin < y x < y.sin
    theorem Real.arcsin_lt_iff_lt_sin' {x : } {y : } (hy : y Set.Ioc (-(Real.pi / 2)) (Real.pi / 2)) :
    x.arcsin < y x < y.sin
    theorem Real.lt_arcsin_iff_sin_lt {x : } {y : } (hx : x Set.Icc (-(Real.pi / 2)) (Real.pi / 2)) (hy : y Set.Icc (-1) 1) :
    x < y.arcsin x.sin < y
    theorem Real.lt_arcsin_iff_sin_lt' {x : } {y : } (hx : x Set.Ico (-(Real.pi / 2)) (Real.pi / 2)) :
    x < y.arcsin x.sin < y
    theorem Real.arcsin_eq_iff_eq_sin {x : } {y : } (hy : y Set.Ioo (-(Real.pi / 2)) (Real.pi / 2)) :
    x.arcsin = y x = y.sin
    @[simp]
    theorem Real.arcsin_nonneg {x : } :
    0 x.arcsin 0 x
    @[simp]
    theorem Real.arcsin_nonpos {x : } :
    x.arcsin 0 x 0
    @[simp]
    theorem Real.arcsin_eq_zero_iff {x : } :
    x.arcsin = 0 x = 0
    @[simp]
    theorem Real.zero_eq_arcsin_iff {x : } :
    0 = x.arcsin x = 0
    @[simp]
    theorem Real.arcsin_pos {x : } :
    0 < x.arcsin 0 < x
    @[simp]
    theorem Real.arcsin_lt_zero {x : } :
    x.arcsin < 0 x < 0
    @[simp]
    theorem Real.arcsin_lt_pi_div_two {x : } :
    x.arcsin < Real.pi / 2 x < 1
    @[simp]
    theorem Real.neg_pi_div_two_lt_arcsin {x : } :
    -(Real.pi / 2) < x.arcsin -1 < x
    @[simp]
    theorem Real.arcsin_eq_pi_div_two {x : } :
    x.arcsin = Real.pi / 2 1 x
    @[simp]
    theorem Real.pi_div_two_eq_arcsin {x : } :
    Real.pi / 2 = x.arcsin 1 x
    @[simp]
    theorem Real.pi_div_two_le_arcsin {x : } :
    Real.pi / 2 x.arcsin 1 x
    @[simp]
    theorem Real.arcsin_eq_neg_pi_div_two {x : } :
    x.arcsin = -(Real.pi / 2) x -1
    @[simp]
    theorem Real.neg_pi_div_two_eq_arcsin {x : } :
    -(Real.pi / 2) = x.arcsin x -1
    @[simp]
    theorem Real.arcsin_le_neg_pi_div_two {x : } :
    x.arcsin -(Real.pi / 2) x -1
    @[simp]
    theorem Real.pi_div_four_le_arcsin {x : } :
    Real.pi / 4 x.arcsin 2 / 2 x

    Real.sin as a PartialHomeomorph between (-π / 2, π / 2) and (-1, 1).

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      theorem Real.cos_arcsin_nonneg (x : ) :
      0 x.arcsin.cos
      theorem Real.cos_arcsin (x : ) :
      x.arcsin.cos = (1 - x ^ 2).sqrt
      theorem Real.tan_arcsin (x : ) :
      x.arcsin.tan = x / (1 - x ^ 2).sqrt
      noncomputable def Real.arccos (x : ) :

      Inverse of the cos function, returns values in the range 0 ≤ arccos x and arccos x ≤ π. It defaults to π on (-∞, -1) and to 0 to (1, ∞).

      Equations
      Instances For
        theorem Real.arccos_eq_pi_div_two_sub_arcsin (x : ) :
        x.arccos = Real.pi / 2 - x.arcsin
        theorem Real.arcsin_eq_pi_div_two_sub_arccos (x : ) :
        x.arcsin = Real.pi / 2 - x.arccos
        theorem Real.arccos_le_pi (x : ) :
        x.arccos Real.pi
        theorem Real.arccos_nonneg (x : ) :
        0 x.arccos
        @[simp]
        theorem Real.arccos_pos {x : } :
        0 < x.arccos x < 1
        theorem Real.cos_arccos {x : } (hx₁ : -1 x) (hx₂ : x 1) :
        x.arccos.cos = x
        theorem Real.arccos_cos {x : } (hx₁ : 0 x) (hx₂ : x Real.pi) :
        x.cos.arccos = x
        theorem Real.arccos_eq_of_eq_cos {x : } {y : } (hy₀ : 0 y) (hy₁ : y Real.pi) (hxy : x = y.cos) :
        x.arccos = y
        theorem Real.arccos_inj {x : } {y : } (hx₁ : -1 x) (hx₂ : x 1) (hy₁ : -1 y) (hy₂ : y 1) :
        x.arccos = y.arccos x = y
        @[simp]
        @[simp]
        theorem Real.arccos_neg_one :
        (-1).arccos = Real.pi
        @[simp]
        theorem Real.arccos_eq_zero {x : } :
        x.arccos = 0 1 x
        @[simp]
        theorem Real.arccos_eq_pi_div_two {x : } :
        x.arccos = Real.pi / 2 x = 0
        @[simp]
        theorem Real.arccos_eq_pi {x : } :
        x.arccos = Real.pi x -1
        theorem Real.arccos_neg (x : ) :
        (-x).arccos = Real.pi - x.arccos
        theorem Real.arccos_of_one_le {x : } (hx : 1 x) :
        x.arccos = 0
        theorem Real.arccos_of_le_neg_one {x : } (hx : x -1) :
        x.arccos = Real.pi
        theorem Real.sin_arccos (x : ) :
        x.arccos.sin = (1 - x ^ 2).sqrt
        @[simp]
        theorem Real.arccos_le_pi_div_two {x : } :
        x.arccos Real.pi / 2 0 x
        @[simp]
        theorem Real.arccos_lt_pi_div_two {x : } :
        x.arccos < Real.pi / 2 0 < x
        @[simp]
        theorem Real.arccos_le_pi_div_four {x : } :
        x.arccos Real.pi / 4 2 / 2 x
        theorem Real.tan_arccos (x : ) :
        x.arccos.tan = (1 - x ^ 2).sqrt / x
        theorem Real.arccos_eq_arcsin {x : } (h : 0 x) :
        x.arccos = (1 - x ^ 2).sqrt.arcsin
        theorem Real.arcsin_eq_arccos {x : } (h : 0 x) :
        x.arcsin = (1 - x ^ 2).sqrt.arccos