leanprover-community / mathlib

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

Zulip Chat Archive

Stream: mathlib4

Topic: Unecessarily complex goal


Eric Wieser (Nov 06 2023 at 11:20):

Guess what the goal is at this sorry?

import Mathlib

example (z : ℤ) : |(z : ℝ)| ≤ z := by
  simp
  sorry

Complex.abs ↑z ≤ ↑z, due to docs#Complex.int_cast_abs / docs3#complex.int_cast_abs


Last updated: May 02 2025 at 03:31 UTC

Theme Simple by wildflame © 2016 Powered by jekyll