Zulip Chat Archive
Stream: new members
Topic: Easiest way to play with casts in C
Srivatsa Srinivas (Feb 06 2025 at 00:33):
Hi all,
What is the easiest way to deal with this minimal working example?
example (a b c : ℝ) : (↑a = (2 : ℂ) * ↑b * ↑c) ↔ (a = 2 *b *c) := by sorry
Best,
Vatsa
Aaron Liu (Feb 06 2025 at 00:48):
import Mathlib
example (a b c : ℝ) : (↑a = (2 : ℂ) * ↑b * ↑c) ↔ (a = 2 *b *c) := by norm_cast
Srivatsa Srinivas (Feb 06 2025 at 00:52):
Thanks!
Last updated: May 02 2025 at 03:31 UTC