Zulip Chat Archive

Stream: Lean for Scientists and Engineers 2024

Topic: MoP 1.2.4


Tyler Josephson ⚛️ (Jul 10 2024 at 18:58):

Illustrating how to ask Lean questions on Zulip

Tyler Josephson ⚛️ (Jul 10 2024 at 18:58):

#mwe and #backticks

Tyler Josephson ⚛️ (Jul 10 2024 at 19:01):

import Mathlib

example {a b c d e f : } (h1 : a * d = b * c) (h2 : c * f = d * e) :
    d * (a * f - b * e) = 0 :=
  calc
    d * (a * f - b * e) = (a * d) * f - b * d * e := by ring
    _ = (b * c) * f - b * (c * f) := by rw [h1,h2]
    _ = 0 := by ring

This is having a problem with the rw line

Tyler Josephson ⚛️ (Jul 10 2024 at 19:02):

Gonzalo saw the issue, the parentheses should be d * (a * f - b * e) = (a*d)*f-(d*e)*b


Last updated: May 02 2025 at 03:31 UTC