Zulip Chat Archive

Stream: new members

Topic: simple problem


BANGJI HU (Sep 17 2024 at 00:21):

import Mathlib.Data.Real.Cardinality
import Mathlib



theorem problem5 {x y : } (h1 : 2  x  2  y) (h2 : x ^ 2 + y ^ 2 = 4) :
    x ^ 2 * y ^ 2 = 0 := by
  apply le_antisymm
  obtain h1 | h2 := h1
  have h3 :=
  calc
    x ^ 2 = 4 - y^2 := by rw [ h2]
    _ = 4 - 0^2 := by rw [h2]
    _  4 := by rw [h2]
  cancel 2 at h3
  calc
    y ^ 2 = 4 - x^2 := by ring
    _ = 4 - 0^2 := by rw[h1]
    _  4 := by numbers
  cancel 2 at h3

BANGJI HU (Sep 17 2024 at 00:22):

seem to be some mistake

Heather Macbeth (Sep 17 2024 at 00:40):

Hi @hand bob, could you please

  1. not double-post
  2. not ask about homework problems from my current course until the week after they are due?

Heather Macbeth (Sep 17 2024 at 00:43):

(I'm not sure how you encountered this problem, but it did not exist on the internet until 5 days ago when I made it up for my homework.)

BANGJI HU (Sep 17 2024 at 00:55):

import Mathlib.Data.Real.Cardinality

import Mathlib


theorem problem5 {x y : } (h1 : 2  x  2  y) (h2 : x ^ 2 + y ^ 2 = 4) :
    x ^ 2 * y ^ 2 = 0 := by
  apply le_antisymm
  obtain h1 | h2 := h1
  have h3 :=
  calc
    x ^ 2 = 4 - y^2 := by rw [ h2]
    _ = 4 - 0^2 := by rw [h2]
    _  4 := by rw [h2]
  simp only [ge_iff_le]
  calc
    y ^ 2 = 4 - x^2 := by ring
    _ = 4 - 0^2 := by rw[h1]
    _  4 := by

BANGJI HU (Sep 17 2024 at 00:56):

can you give me some hint

BANGJI HU (Sep 17 2024 at 00:56):

@Heather Macbeth

Heather Macbeth (Sep 17 2024 at 00:58):

@hand bob If you are one of my students, please email me directly! If not, please wait a few days, and then post here again (and explain your question more precisely).


Last updated: May 02 2025 at 03:31 UTC