aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Rtrigo_calc.v
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2018-06-22 13:45:03 +0200
committerGravatar Maxime Dénès <mail@maximedenes.fr>2018-07-17 14:15:59 +0200
commit8c43e795c772090b336c0f170a6e5dcab196125d (patch)
tree98508f7e342142dd017da56872f74df73e6fce58 /theories/Reals/Rtrigo_calc.v
parentb799252775563b4f46f5ea39cbfc469759e7a296 (diff)
Remove fourier plugin
As stated in the manual, the fourier tactic is subsumed by lra.
Diffstat (limited to 'theories/Reals/Rtrigo_calc.v')
-rw-r--r--theories/Reals/Rtrigo_calc.v1
1 files changed, 0 insertions, 1 deletions
diff --git a/theories/Reals/Rtrigo_calc.v b/theories/Reals/Rtrigo_calc.v
index 7cbfc6303..78797c87c 100644
--- a/theories/Reals/Rtrigo_calc.v
+++ b/theories/Reals/Rtrigo_calc.v
@@ -205,7 +205,6 @@ Proof with trivial.
rewrite cos2; unfold Rsqr; rewrite sin_PI6; rewrite sqrt_def...
field.
left ; prove_sup0.
- discrR.
Qed.
Lemma tan_PI6 : tan (PI / 6) = 1 / sqrt 3.