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/Basic_mathd_algebra_513/mathd_algebra_513_prover.lean b/EasyLean/Basic_mathd_algebra_513/mathd_algebra_513_prover.lean new file mode 100644 index 0000000..8b2fe85 --- /dev/null +++ b/EasyLean/Basic_mathd_algebra_513/mathd_algebra_513_prover.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 + constructor + · linarith [h₀, h₁] + · linarith [h₀, h₁] + + diff --git a/build_filtered.sh b/build_filtered.sh new file mode 100644 index 0000000..7e82dc1 --- /dev/null +++ b/build_filtered.sh @@ -0,0 +1,29 @@ +#!/bin/bash + +echo "Running lake build (quiet mode, errors only)..." + +# Run lake build with --quiet, capture output and exit code +OUTPUT=$(lake exe cache get && lake build --quiet 2>&1) +EXIT_CODE=$? + +# Count errors and warnings +ERROR_COUNT=$(echo "$OUTPUT" | grep -c "^error:" || true) +WARNING_COUNT=$(echo "$OUTPUT" | grep -c "^warning:" || true) + +echo "════════════════════════════════════════════════" +echo "Build Summary:" +echo " Warnings: $WARNING_COUNT (suppressed in output below)" +echo " Errors: $ERROR_COUNT" +echo " Exit code: $EXIT_CODE" +echo "════════════════════════════════════════════════" + +if [ $EXIT_CODE -ne 0 ]; then + echo "" + echo "❌ BUILD FAILED - Showing errors only:" + echo "" + echo "$OUTPUT" | grep -A 3 "^error:" +else + echo "✅ BUILD SUCCEEDED" +fi + +exit $EXIT_CODE