src/HOL/Transcendental.thy
changeset 62393 a620a8756b7c
parent 62381 a6479cb85944
parent 62390 842917225d56
child 62679 092cb9c96c99
equal deleted inserted replaced
62385:7891843d79bb 62393:a620a8756b7c
  4263 lemma tan_pos_pi2_le: "0 \<le> x ==> x < pi/2 \<Longrightarrow> 0 \<le> tan x"
  4263 lemma tan_pos_pi2_le: "0 \<le> x ==> x < pi/2 \<Longrightarrow> 0 \<le> tan x"
  4264   using less_eq_real_def tan_gt_zero by auto
  4264   using less_eq_real_def tan_gt_zero by auto
  4265 
  4265 
  4266 lemma cos_tan: "\<bar>x\<bar> < pi/2 \<Longrightarrow> cos(x) = 1 / sqrt(1 + tan(x) ^ 2)"
  4266 lemma cos_tan: "\<bar>x\<bar> < pi/2 \<Longrightarrow> cos(x) = 1 / sqrt(1 + tan(x) ^ 2)"
  4267   using cos_gt_zero_pi [of x]
  4267   using cos_gt_zero_pi [of x]
  4268   by (simp add: divide_simps tan_def real_sqrt_divide abs_if split: split_if_asm)
  4268   by (simp add: divide_simps tan_def real_sqrt_divide abs_if split: if_split_asm)
  4269 
  4269 
  4270 lemma sin_tan: "\<bar>x\<bar> < pi/2 \<Longrightarrow> sin(x) = tan(x) / sqrt(1 + tan(x) ^ 2)"
  4270 lemma sin_tan: "\<bar>x\<bar> < pi/2 \<Longrightarrow> sin(x) = tan(x) / sqrt(1 + tan(x) ^ 2)"
  4271   using cos_gt_zero [of "x"] cos_gt_zero [of "-x"]
  4271   using cos_gt_zero [of "x"] cos_gt_zero [of "-x"]
  4272   by (force simp add: divide_simps tan_def real_sqrt_divide abs_if split: split_if_asm)
  4272   by (force simp add: divide_simps tan_def real_sqrt_divide abs_if split: if_split_asm)
  4273 
  4273 
  4274 lemma tan_mono_le: "-(pi/2) < x ==> x \<le> y ==> y < pi/2 \<Longrightarrow> tan(x) \<le> tan(y)"
  4274 lemma tan_mono_le: "-(pi/2) < x ==> x \<le> y ==> y < pi/2 \<Longrightarrow> tan(x) \<le> tan(y)"
  4275   using less_eq_real_def tan_monotone by auto
  4275   using less_eq_real_def tan_monotone by auto
  4276 
  4276 
  4277 lemma tan_mono_lt_eq: "-(pi/2) < x ==> x < pi/2 ==> -(pi/2) < y ==> y < pi/2
  4277 lemma tan_mono_lt_eq: "-(pi/2) < x ==> x < pi/2 ==> -(pi/2) < y ==> y < pi/2
  4282          \<Longrightarrow> (tan(x) \<le> tan(y) \<longleftrightarrow> x \<le> y)"
  4282          \<Longrightarrow> (tan(x) \<le> tan(y) \<longleftrightarrow> x \<le> y)"
  4283   by (meson tan_mono_le not_le tan_monotone)
  4283   by (meson tan_mono_le not_le tan_monotone)
  4284 
  4284 
  4285 lemma tan_bound_pi2: "\<bar>x\<bar> < pi/4 \<Longrightarrow> \<bar>tan x\<bar> < 1"
  4285 lemma tan_bound_pi2: "\<bar>x\<bar> < pi/4 \<Longrightarrow> \<bar>tan x\<bar> < 1"
  4286   using tan_45 tan_monotone [of x "pi/4"] tan_monotone [of "-x" "pi/4"]
  4286   using tan_45 tan_monotone [of x "pi/4"] tan_monotone [of "-x" "pi/4"]
  4287   by (auto simp: abs_if split: split_if_asm)
  4287   by (auto simp: abs_if split: if_split_asm)
  4288 
  4288 
  4289 lemma tan_cot: "tan(pi/2 - x) = inverse(tan x)"
  4289 lemma tan_cot: "tan(pi/2 - x) = inverse(tan x)"
  4290   by (simp add: tan_def sin_diff cos_diff)
  4290   by (simp add: tan_def sin_diff cos_diff)
  4291 
  4291 
  4292 subsection \<open>Cotangent\<close>
  4292 subsection \<open>Cotangent\<close>