Skip to content

Commit b9c61b4

Browse files
committed
Update tests
1 parent 9f8eda8 commit b9c61b4

File tree

4 files changed

+8
-6
lines changed

4 files changed

+8
-6
lines changed

tests/lean/1038.lean.expected.out

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
1038.lean:1:7-1:21: error(lean.unknownIdentifier): Unknown constant `IO.FS.realpath`
1+
1038.lean:1:10-1:12: error(lean.unknownIdentifier): Unknown constant `IO.FS.realpath`

tests/lean/346.lean.expected.out

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1,5 +1,5 @@
1-
346.lean:10:6-10:16: error(lean.unknownIdentifier): Unknown constant `SomeType.b`
2-
346.lean:13:2-13:5: error: Invalid field `z`: The environment does not contain `Nat.z`
1+
346.lean:10:15-10:16: error(lean.unknownIdentifier): Unknown constant `SomeType.b`
2+
346.lean:13:4-13:5: error: Invalid field `z`: The environment does not contain `Nat.z`
33
x
44
has type
55
Nat
Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -1,5 +1,5 @@
11
funind_errors.lean:4:7-4:26: error(lean.unknownIdentifier): Unknown identifier `doesNotExist.induct`
2-
funind_errors.lean:22:7-22:23: error(lean.unknownIdentifier): Unknown constant `takeWhile.induct`
2+
funind_errors.lean:22:17-22:23: error(lean.unknownIdentifier): Unknown constant `takeWhile.induct`
33
takeWhile.foo.induct.{u_1} {α : Type u_1} (p : α → Bool) (as : Array α) (motive : Nat → Array α → Prop)
44
(case1 :
55
∀ (i : Nat) (r : Array α) (h : i < as.size),
@@ -10,5 +10,5 @@ takeWhile.foo.induct.{u_1} {α : Type u_1} (p : α → Bool) (as : Array α) (mo
1010
have a := as[i];
1111
¬p a = true → motive i r)
1212
(case3 : ∀ (i : Nat) (r : Array α), ¬i < as.size → motive i r) (i : Nat) (r : Array α) : motive i r
13-
funind_errors.lean:38:7-38:20: error(lean.unknownIdentifier): Unknown constant `idEven.induct`
14-
funind_errors.lean:45:7-45:19: error(lean.unknownIdentifier): Unknown constant `idAcc.induct`
13+
funind_errors.lean:38:14-38:20: error(lean.unknownIdentifier): Unknown constant `idEven.induct`
14+
funind_errors.lean:45:13-45:19: error(lean.unknownIdentifier): Unknown constant `idAcc.induct`

tests/lean/run/issue10821.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1,3 +1,5 @@
1+
set_option linter.deprecated true
2+
13
/-!
24
Checks that deprecated names in projection notation cause just
35
the name to be marked, not the whole expression.

0 commit comments

Comments
 (0)