Zulip Chat Archive

Stream: new members

Topic: Numerical computations plus inequalities


André Hernández-Espiet (Rutgers) (Jan 26 2024 at 00:54):

Hi all, I was wondering if there is a tactic sequence that would solve this without prior knowledge of bounds:

import Mathlib.Data.Real.Pi.Bounds

example : 3 * Real.pi < 10 := by
  have h0 : (3.15 : ) * 3 < 10 := by norm_num
  linarith[Real.pi_lt_315]

Kevin Buzzard (Jan 26 2024 at 04:02):

This might be the not-yet-existing by_approx tactic that people have been occasionally discussing.

Yaël Dillies (Jan 26 2024 at 08:20):

Yes, search for approx on Zulip

Mauricio Collares (Jan 26 2024 at 08:49):

by_approx is at #8949


Last updated: May 02 2025 at 03:31 UTC