Zulip Chat Archive

Stream: mathlib4

Topic: norm_cast gives Int.subNatNat


Eric Wieser (Dec 12 2023 at 15:42):

Is this really the behavior we want?

import Mathlib

example (n : ) : (n : ) - 1 = 3 := by
  norm_cast
  /-
  n : ℕ
  ⊢ Int.subNatNat n 1 = 3
  -/
  sorry

Yury G. Kudryashov (Dec 12 2023 at 15:54):

Which lemma does it use?

Ruben Van de Velde (Dec 12 2023 at 16:27):

I thought that was fixed

Ruben Van de Velde (Dec 12 2023 at 16:28):

Ref https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/norm_cast.20leaks.20Int.2EsubSubNat


Last updated: Dec 20 2023 at 11:08 UTC