Skip to content

Commit d0059f7

Browse files
committed
chore: update tests
1 parent 990f9ce commit d0059f7

7 files changed

+14
-14
lines changed

tests/lean/1363.lean.expected.out

Lines changed: 5 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -1,5 +1,5 @@
1-
1363.lean:4:2-4:14: error: invalid use of `[macro_inline]` attribute at `f`, it is not supported in this kind of declaration, declaration must be a non-recursive definition
2-
1363.lean:9:2-9:14: error: invalid use of `[macro_inline]` attribute at `g`, it is not supported in this kind of declaration, declaration must be a non-recursive definition
3-
1363.lean:15:2-15:14: error: invalid use of `[macro_inline]` attribute at `h._unary`, it is not supported in this kind of declaration, declaration must be a non-recursive definition
4-
1363.lean:15:2-15:14: error: invalid use of `[macro_inline]` attribute at `h`, it is not supported in this kind of declaration, declaration must be a non-recursive definition
5-
1363.lean:21:2-21:14: error: invalid use of `[macro_inline]` attribute at `skipMany`, it is not supported in this kind of declaration, declaration must be a non-recursive definition
1+
1363.lean:4:2-4:14: error: Cannot add `[macro_inline]` attribute to `f`: This attribute does not support this kind of declaration; only non-recursive definitions are supported
2+
1363.lean:9:2-9:14: error: Cannot add `[macro_inline]` attribute to `g`: This attribute does not support this kind of declaration; only non-recursive definitions are supported
3+
1363.lean:15:2-15:14: error: Cannot add `[macro_inline]` attribute to `h._unary`: This attribute does not support this kind of declaration; only non-recursive definitions are supported
4+
1363.lean:15:2-15:14: error: Cannot add `[macro_inline]` attribute to `h`: This attribute does not support this kind of declaration; only non-recursive definitions are supported
5+
1363.lean:21:2-21:14: error: Cannot add `[macro_inline]` attribute to `skipMany`: This attribute does not support this kind of declaration; only non-recursive definitions are supported

tests/lean/inductive1.lean.expected.out

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -18,7 +18,7 @@ inductive1.lean:69:2-69:5: error: 'Boo.T1.bla' has already been declared
1818
inductive1.lean:73:10-73:12: error: 'Boo.T1' has already been declared
1919
inductive1.lean:80:0-80:27: error: invalid use of 'partial' in inductive declaration
2020
inductive1.lean:81:0-81:33: error: invalid use of 'noncomputable' in inductive declaration
21-
inductive1.lean:82:2-82:8: error: declaration is not a definition 'T1''
21+
inductive1.lean:82:2-82:8: error: Cannot add attribute `[inline]`: Declaration `T1'` is not a definition
2222
inductive1.lean:85:0-85:17: error: invalid 'private' constructor in a 'private' inductive datatype
2323
inductive1.lean:93:7-93:26: error: invalid inductive type, cannot mix unsafe and safe declarations in mutually inductive datatypes
2424
inductive1.lean:100:0-100:4: error: Missing resulting type for constructor 'T1.z2': Its resulting type must be specified because it is part of an inductive family declaration
Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,4 @@
1-
nonfatalattrs.lean:6:2-6:19: error: unknown attribute [attrUnimplementedattr]
1+
nonfatalattrs.lean:6:2-6:19: error: Unknown attribute `[attrUnimplementedattr]`
22
foo : Nat
33
nonfatalattrs.lean:11:12-11:17: error: invalid 'class', declaration 'bar.bar' must be inductive datatype, structure, or constant
44
bar : Nat

tests/lean/run/3643.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -90,7 +90,7 @@ end Ex2
9090
section Ex3
9191

9292
-- TODO: allow 'scoped' here? The limitation is in attribute processing itself, not the 'ext' attribute.
93-
/-- error: scoped attributes must be used inside namespaces -/
93+
/-- error: Scoped attributes must be used inside namespaces -/
9494
#guard_msgs in
9595
@[scoped ext] structure S3' (α β : Type _) where
9696
a : α

tests/lean/run/reducibilityAttrValidation.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -84,7 +84,7 @@ Note: Use `set_option allowUnsafeReducibility true` to override reducibility sta
8484
#guard_msgs in
8585
attribute [irreducible] Nat.add
8686

87-
/-- error: scoped attributes must be used inside namespaces -/
87+
/-- error: Scoped attributes must be used inside namespaces -/
8888
#guard_msgs in
8989
attribute [scoped reducible] Nat.add
9090

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -1,4 +1,4 @@
1-
scopedInstanceOutsideNamespace.lean:1:0-2:38: error: scoped attributes must be used inside namespaces
1+
scopedInstanceOutsideNamespace.lean:1:0-2:38: error: Scoped attributes must be used inside namespaces
22
"true"
3-
scopedInstanceOutsideNamespace.lean:6:0-6:30: error: scoped attributes must be used inside namespaces
4-
scopedInstanceOutsideNamespace.lean:8:2-8:17: error: scoped attributes must be used inside namespaces
3+
scopedInstanceOutsideNamespace.lean:6:0-6:30: error: Scoped attributes must be used inside namespaces
4+
scopedInstanceOutsideNamespace.lean:8:2-8:17: error: Scoped attributes must be used inside namespaces

tests/lean/scopedMacros.lean.expected.out

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1,10 +1,10 @@
11
10 + 1 : Nat
22
scopedMacros.lean:11:7-11:11: error: unknown identifier 'foo!'
33
10 + 1 : Nat
4-
scopedMacros.lean:19:7-19:50: error: scoped attributes must be used inside namespaces
4+
scopedMacros.lean:19:7-19:50: error: Scoped attributes must be used inside namespaces
55
scopedMacros.lean:19:7-19:50: error: invalid syntax node kind 'termBla!_'
66
scopedMacros.lean:29:7-29:11: error: unknown identifier 'bla!'
7-
scopedMacros.lean:36:7-36:45: error: scoped attributes must be used inside namespaces
7+
scopedMacros.lean:36:7-36:45: error: Scoped attributes must be used inside namespaces
88
10 + 20 : Nat
99
scopedMacros.lean:47:7-47:14: error: elaboration function for 'termBar!_' has not been implemented
1010
bar! 10

0 commit comments

Comments
 (0)