Library Coq.Reals.Rtrigo_facts


Require Import Rbase.
Require Import Rtrigo1.
Require Import Rfunctions.

Require Import Lra.
Require Import Ranalysis_reg.

Local Open Scope R_scope.

Bounds of expressions with trigonometric functions


Lemma sin2_bound : forall x,
  0 <= (sin x <= 1.

Lemma cos2_bound : forall x,
  0 <= (cos x <= 1.

Express trigonometric functions with each other

Express sin and cos with each other


Lemma cos_sin : forall x, cos x >=0 ->
  cos x = sqrt(1 - (sin x).

Lemma cos_sin_opp : forall x, cos x <=0 ->
  cos x = - sqrt(1 - (sin x).

Lemma cos_sin_Rabs : forall x,
  Rabs (cos x) = sqrt(1 - (sin x).

Lemma sin_cos : forall x, sin x >=0 ->
  sin x = sqrt(1 - (cos x).

Lemma sin_cos_opp : forall x, sin x <=0 ->
  sin x = - sqrt(1 - (cos x).

Lemma sin_cos_Rabs : forall x,
  Rabs (sin x) = sqrt(1 - (cos x).

Express tan with sin and cos


Lemma tan_sin : forall x, 0 <= cos x ->
  tan x = sin x / sqrt (1 - (sin x).

Lemma tan_sin_opp : forall x, 0 > cos x ->
  tan x = - (sin x / sqrt (1 - (sin x)).

Note: tan_sin_Rabs wouldn't make a lot of sense, because one would need Rabs on both sides

Lemma tan_cos : forall x, 0 <= sin x ->
  tan x = sqrt (1 - (cos x) / cos x.

Lemma tan_cos_opp : forall x, 0 >= sin x ->
  tan x = - sqrt (1 - (cos x) / cos x.

Express sin and cos with tan


Lemma sin_tan : forall x, 0 < cos x ->
  sin x = tan x / sqrt (1 + (tan x).

Lemma cos_tan : forall x, 0 < cos x ->
  cos x = 1 / sqrt (1 + (tan x).

Additional shift lemmas for sin, cos, tan


Lemma sin_pi_minus : forall x,
  sin (PI - x) = sin x.

Lemma sin_pi_plus : forall x,
  sin (PI + x) = - sin x.

Lemma cos_pi_minus : forall x,
  cos (PI - x) = - cos x.

Lemma cos_pi_plus : forall x,
  cos (PI + x) = - cos x.

Lemma tan_pi_minus : forall x, cos x <> 0 ->
  tan (PI - x) = - tan x.

Lemma tan_pi_plus : forall x, cos x <> 0 ->
  tan (PI + x) = tan x.