Zulip Chat Archive

Stream: general

Topic: norm_num splits multiplication equality


Yaël Dillies (Dec 18 2023 at 15:10):

@Mario Carneiro, I just uncovered a minor bug in norm_num. It seems to apply docs#mul_eq_mul_right_iff under the hood, even though that's not in its specification:

import Mathlib.Tactic.NormNum

example (a b c : ) : 4096 * a * c = 512 * 8 * b * c := by
  norm_num
-- Expected:
/-
unsolved goals
a b c : ℕ
⊢ 4096 * a * c = 4096 * b * c
-/
-- Actual:
/-
unsolved goals
a b c : ℕ
⊢ a = b ∨ c = 0
-/

Eric Rodriguez (Dec 18 2023 at 15:13):

It's a simp lemma, norm_num runs simp

Eric Rodriguez (Dec 18 2023 at 15:13):

norm_num1 won't


Last updated: Dec 20 2023 at 11:08 UTC