Skip to content

Commit

Permalink
cleanup tests
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed May 6, 2024
1 parent 68ddd10 commit 683fa0c
Show file tree
Hide file tree
Showing 2 changed files with 1 addition and 3 deletions.
2 changes: 0 additions & 2 deletions test/Mathlib/test/20240209.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,2 @@
import Std.Tactic.Simpa

example : False := by
simpa using show False by done
2 changes: 1 addition & 1 deletion test/Mathlib/test/H20231214.lean
Original file line number Diff line number Diff line change
Expand Up @@ -27,4 +27,4 @@ theorem mathd_algebra_35
have hQ : ∀ x, p x = 6 / x := by
intro x
calc p x = 6 / x * p x := h₀ (x)
_ = (6/2) * 6 / x * (6 / x) := sub_sub_sub_cancel sq_ne_zero
_ = (6/2) * 6 / x * (6 / x) := sorry

0 comments on commit 683fa0c

Please sign in to comment.