diff --git a/EasyLean/Basic.lean b/EasyLean/Basic.lean index 305e1ca..5a1d082 100644 --- a/EasyLean/Basic.lean +++ b/EasyLean/Basic.lean @@ -1,12 +1,2 @@ -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 +import EasyLean.Theorems.MathdAlgebra513 +import EasyLean.Theorems.EqFour diff --git a/EasyLean/Theorems/EqFour.lean b/EasyLean/Theorems/EqFour.lean new file mode 100644 index 0000000..771eb48 --- /dev/null +++ b/EasyLean/Theorems/EqFour.lean @@ -0,0 +1,4 @@ +import Mathlib + +theorem eq_four (a b c d : Nat) (hab : a = b) (had : a = d) (hac : a = c) : c = b := by + exact hac.symm.trans hab diff --git a/EasyLean/Theorems/MathdAlgebra513.lean b/EasyLean/Theorems/MathdAlgebra513.lean new file mode 100644 index 0000000..34ea1ca --- /dev/null +++ b/EasyLean/Theorems/MathdAlgebra513.lean @@ -0,0 +1,8 @@ +import Mathlib + +theorem mathd_algebra_513 (a b : ℝ) (h₀ : 3 * a + 2 * b = 5) (h₁ : a + b = 2) : a = 1 ∧ b = 1 := by + have ha : a = 1 := by + linarith [h₀, h₁] + have hb : b = 1 := by + linarith [h₀, h₁] + exact ⟨ha, hb⟩