Zulip Chat Archive
Stream: maths
Topic: norm_num question and comment
Kevin Buzzard (Aug 13 2018 at 20:30):
import data.real.basic import tactic.norm_num definition A : set ℝ := { x | x ^ 2 < 3} -- hangs --example : (1 / 2 : ℝ) ∈ A := by norm_num example : (1 / 2 : ℝ) ^ 2 < 3 ∧ (1 / 2) ^ 2 < 4 := begin split, -- two goals norm_num, -- where did my second goal go? end
I don't really know why the first example hangs. I can believe that Lean is reluctant to change (1/2) \in A
to A (1/2)
to (lam x, x^2<3) (1/2)
to (1/2)^2<3
(note that norm_num can solve the latter no problem) but I don't really know why it hangs. The reason I discovered it choked on this was trying to solve a goal of the form (1 / 2 : ℝ) ^ 2 < 3 ∧ (1 / 2 : ℝ) ∈ A
by "split,norm_num,..." and norm_num
hung on me, I thought because of the first goal, but actually because of the second.
Is making norm_num
just act on the current goal something that can be trivially done? I know about the {norm_num}
trick but this was an undergraduate that tripped up, not me.
Last updated: Dec 20 2023 at 11:08 UTC