Skip to content

Commit

Permalink
fixes
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Dec 22, 2023
1 parent d6b392a commit ea3474d
Show file tree
Hide file tree
Showing 3 changed files with 19 additions and 0 deletions.
1 change: 1 addition & 0 deletions test/Mathlib/ReplMathlibTests.lean
Original file line number Diff line number Diff line change
@@ -0,0 +1 @@
import Mathlib
2 changes: 2 additions & 0 deletions test/Mathlib/lakefile.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,5 +5,7 @@ package «repl-mathlib-tests» where
-- add package configuration options here
require mathlib from git "https://github.com/leanprover-community/mathlib4" @ "master"

@[default_target]
lean_lib «ReplMathlibTests» where
globs := #[.submodules `test]
-- add library configuration options here
16 changes: 16 additions & 0 deletions test/Mathlib/test/H20231214.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,6 +3,22 @@ open Real
open Nat
open BigOperators

/--
error: type mismatch
h₀ x
has type
p x = 2 - x ^ 2 : Prop
but is expected to have type
p x = 6 / x * p x : Prop
---
error: unsolved goals
p q : ℝ → ℝ
h₀ : ∀ (x : ℝ), p x = 2 - x ^ 2
h₁ : ∀ (x : ℝ), x ≠ 0 → q x = 6 / x
hQ : ∀ (x : ℝ), p x = 6 / x
⊢ p (q 2) = -7
-/
#guard_msgs in
theorem mathd_algebra_35
(p q : ℝ → ℝ)
(h₀ : ∀ x, p x = 2 - x^2)
Expand Down

0 comments on commit ea3474d

Please sign in to comment.