Zulip Chat Archive
Stream: maths
Topic: A question about getting a map
Junqi Liu (Jul 11 2024 at 07:05):
If I have such lemma
lemma P {f : ℕ → ℝ} (r : ℕ) : ∃ a : ℤ, r = a / f r := by sorry
How can I get a map which maps to in lemma P?
Kevin Buzzard (Jul 11 2024 at 07:16):
In tactic mode you can use the choose
tactic and in term mode you can use (P r).choose
for the function and (P r).choose_spec
for the equality defining the function.
Junqi Liu (Jul 11 2024 at 08:52):
oh! Cool! I have solved my sorry by your suggestion! Thanks a lot!
Last updated: May 02 2025 at 03:31 UTC