Skip to content

Instantly share code, notes, and snippets.

@satos---jp
Created May 26, 2014 11:42
Show Gist options
  • Save satos---jp/4221f860dbaa86612259 to your computer and use it in GitHub Desktop.
Save satos---jp/4221f860dbaa86612259 to your computer and use it in GitHub Desktop.
Require Import Reals.
Require Import Fourier.
Theorem PI_RGT_3_05 : (PI > 3 + 5/100)%R.
Proof.
assert (((sum_f_R0 (tg_alt PI_tg) (S (2 * 5)))%R <= (PI / 4)%R <=
(sum_f_R0 (tg_alt PI_tg) (2 * 5))%R)%R).
apply PI_ineq.
simpl H.
destruct H.
assert (((sum_f_R0 (tg_alt PI_tg) (S(2 * 5)))*4)<=PI).
assert (PI = PI/4*4).
field.
rewrite H1.
apply Rmult_le_compat_r.
fourier.
apply H.
apply (Rge_gt_trans PI (sum_f_R0 (tg_alt PI_tg) (S (2 * 5)) * 4 ) (3 + 5 / 100)).
fourier.
simpl.
unfold tg_alt.
unfold PI_tg.
unfold INR.
simpl.
field_simplify.
apply Rminus_gt.
field_simplify.
assert (0/1 = 0).
field.
rewrite H2.
prove_sup.
apply Rinv_0_lt_compat.
prove_sup.
Qed.
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment