Skip to content

Commit 23d879d

Browse files
committed
really fix tests
1 parent e459aaf commit 23d879d

File tree

2 files changed

+4
-4
lines changed

2 files changed

+4
-4
lines changed

tests/lean/run/derivingBEqLinear.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -38,7 +38,7 @@ info: instBEqL.beq_spec.{u_1} {α✝ : Type u_1} [BEq α✝] (x✝ x✝¹ : L α
3838
match x✝, x✝¹, h with
3939
| L.nil, L.nil, ⋯ => true
4040
| L.cons a a_1, L.cons a' a'_1, ⋯ => a == a' && a_1 == a'_1
41-
| { decide := false, reflects_decide := h } => false
41+
| { decide := false, reflects_decide := reflects_decide } => false
4242
-/
4343
#guard_msgs in #check instBEqL.beq_spec
4444

@@ -69,7 +69,7 @@ info: theorem InNamespace.instBEqL'.beq_spec.{u_1} : ∀ {α : Type u_1} [inst :
6969
match x, x_1, h with
7070
| InNamespace.L'.nil, InNamespace.L'.nil, ⋯ => true
7171
| InNamespace.L'.cons a a_1, InNamespace.L'.cons a' a'_1, ⋯ => a == a' && a_1 == a'_1
72-
| { decide := false, reflects_decide := h } => false
72+
| { decide := false, reflects_decide := reflects_decide } => false
7373
-/
7474
#guard_msgs in #print sig InNamespace.instBEqL'.beq_spec
7575

@@ -86,7 +86,7 @@ info: instBEqVec.beq_spec.{u_1} {α✝ : Type u_1} {a✝ : Nat} [BEq α✝] (x
8686
match a✝, x✝, x✝¹ with
8787
| 0, Vec.nil, Vec.nil, ⋯ => true
8888
| x + 1, Vec.cons a a_1, Vec.cons a' a'_1, ⋯ => a == a' && a_1 == a'_1
89-
| { decide := false, reflects_decide := h } => false
89+
| { decide := false, reflects_decide := reflects_decide } => false
9090
-/
9191
#guard_msgs in
9292
#check instBEqVec.beq_spec

tests/lean/run/reduceBEqSimproc.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -35,7 +35,7 @@ info: Linear.instBEqL.beq.eq_1.{u_1} {α✝ : Type u_1} [BEq α✝] (x✝ x✝¹
3535
match x✝, x✝¹, h with
3636
| L.nil, L.nil, ⋯ => true
3737
| L.cons a a_1, L.cons a' a'_1, ⋯ => a == a' && instBEqL.beq a_1 a'_1
38-
| { decide := false, reflects_decide := h } => false
38+
| { decide := false, reflects_decide := reflects_decide } => false
3939
-/
4040
#guard_msgs in
4141
#check instBEqL.beq.eq_1

0 commit comments

Comments
 (0)