diff --git a/EasyLean.lean b/EasyLean.lean index a53489d..5b5278b 100644 --- a/EasyLean.lean +++ b/EasyLean.lean @@ -1 +1,2 @@ import EasyLean.Basic +import EasyLean.ProblemArchive.mathd_algebra_513 diff --git a/EasyLean/Basic.lean b/EasyLean/Basic.lean index 305e1ca..5c0c53b 100644 --- a/EasyLean/Basic.lean +++ b/EasyLean/Basic.lean @@ -1,12 +1,5 @@ import Mathlib.Data.Real.Basic import Mathlib.Tactic.Linarith -theorem mathd_algebra_513 - (a b : ℝ) - (h₀ : 3 * a + 2 * b = 5) - (h₁ : a + b = 2) : - a = 1 ∧ b = 1 := by - sorry - theorem eq_four : ∀ a b c d : Nat, a = b → a = d → a = c → c = b := by sorry diff --git a/EasyLean/ProblemArchive/mathd_algebra_513.lean b/EasyLean/ProblemArchive/mathd_algebra_513.lean new file mode 100644 index 0000000..fca4307 --- /dev/null +++ b/EasyLean/ProblemArchive/mathd_algebra_513.lean @@ -0,0 +1,7 @@ +import Mathlib.Data.Real.Basic +import Mathlib.Tactic.Linarith + +theorem mathd_algebra_513 (a b : ℝ) (h₀ : 3 * a + 2 * b = 5) (h₁ : a + b = 2) : a = 1 ∧ b = 1 := by + constructor + · linarith [h₀, h₁] + · linarith [h₀, h₁]