leanprover-community / mathlib

  • Home
  • Zulip archive
  • API documentation
  • Lean web editor
  • Links

Zulip Chat Archive

Stream: mathlib4

Topic: ring regression in v4.19.0-rc2


Yaël Dillies (Apr 09 2025 at 17:14):

The following used to work. Since bumping to v.4.19.0-rc2 (or around), it doesn't.

import Mathlib.Tactic.Ring

example (ε : ℚ) (n : ℕ) : (ε / 2) ^ n = ε ^ n / 2 ^ n := by ring

Yaël Dillies (Apr 09 2025 at 17:15):

It looks like the / 2 in the LHS becomes the 1 / 2, while the one in the RHS becomes the atom 2⁻¹


Last updated: May 02 2025 at 03:31 UTC

Theme Simple by wildflame © 2016 Powered by jekyll