Pantograph/experiments/dsp/lean_src_proj/MATH/algebra_683.lean

20 lines
1.0 KiB
Plaintext
Raw Blame History

This file contains ambiguous Unicode characters

This file contains Unicode characters that might be confused with other characters. If you think that this is intentional, you can safely ignore this warning. Use the Escape button to reveal them.

-- {
-- "problem": "If $\\sqrt{2\\sqrt{t-2}} = \\sqrt[4]{7 - t}$, then find $t$.",
-- "level": "Level 4",
-- "type": "Algebra",
-- "solution": "We raise both sides to the fourth power, which is equivalent to squaring twice, in order to get rid of the radicals. The left-hand side becomes $$\\left(\\sqrt{2\\sqrt{t-2}}\\right)^4 = \\left(2\\sqrt{t-2}\\right)^2 = 4 \\cdot (t-2) = 4t-8.$$The right-hand side becomes $\\left(\\sqrt[4]{7-t}\\right)^4 = 7-t$. Setting them equal, $$4t-8 = 7-t \\quad\\Longrightarrow\\quad 5t = 15,$$and $t = \\boxed{3}$. Checking, we find that this value does indeed satisfy the original equation."
-- }
import Mathlib.Data.Real.Basic
import Mathlib.Data.Nat.Pow
noncomputable def a (t : ) : := (2 * (t - 2) ^ (1 / 2)) ^ (1/2)
noncomputable def b (t : ) : := (7 - t)^(1/4)
def valid_t (t : ) : Prop :=
a t = b t
theorem LHS_to_4 : ∀ t : , (a t) ^ 4 = 4 * t - 8 := by sorry
theorem RHS_to_4 : ∀ t : , (b t) ^ 4 = 7 - t := by sorry
theorem solution : valid_t 3 := by sorry