Skip to content

Commit b5a509b

Browse files
committed
fix test
1 parent 198d368 commit b5a509b

File tree

1 file changed

+61
-3
lines changed

1 file changed

+61
-3
lines changed

tests/lean/815b.lean.expected.out

Lines changed: 61 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -24,7 +24,7 @@
2424
Transformer
2525
fun redf a => redf
2626
[Meta.synthInstance] new goal IsSmooth f
27-
[Meta.synthInstance.instances] #[inst✝]
27+
[Meta.synthInstance.instances] #[@identity, @const, @parm, @comp, @diag, @swap, inst✝]
2828
[Meta.synthInstance] ✅️ apply inst✝ to IsSmooth f
2929
[Meta.synthInstance.tryResolve] ✅️ IsSmooth f ≟ IsSmooth f
3030
[Meta.synthInstance.answer] ✅️ IsSmooth f
@@ -44,17 +44,75 @@
4444
Transformer
4545
fun redf a => redf
4646
[Meta.synthInstance] new goal ∀ (b : β), IsSmooth (f b)
47-
[Meta.synthInstance.instances] #[inst✝]
47+
[Meta.synthInstance.instances] #[@identity, @const, @parm, @comp, @diag, inst✝]
4848
[Meta.synthInstance] ❌️ apply inst✝ to ∀ (b : β), IsSmooth (f b)
4949
[Meta.synthInstance.tryResolve] ❌️ IsSmooth (f b) ≟ IsSmooth f
50+
[Meta.synthInstance] ✅️ apply @diag to ∀ (b : β), IsSmooth (f b)
51+
[Meta.synthInstance.tryResolve] ✅️ IsSmooth (f b) ≟ IsSmooth fun a => f b a
52+
[Meta.synthInstance.unusedArgs] ∀ (b : β), IsSmooth f
53+
has unused arguments, reduced type
54+
IsSmooth f
55+
Transformer
56+
fun redf b => redf
57+
[Meta.synthInstance.resume] propagating ∀ (b : β),
58+
IsSmooth f to subgoal ∀ (b : β), IsSmooth f of ∀ (b : β), IsSmooth (f b)
59+
[Meta.synthInstance.resume] size: 1
60+
[Meta.synthInstance.unusedArgs] ∀ (b b : β), IsSmooth (f b)
61+
has unused arguments, reduced type
62+
∀ (b : β), IsSmooth (f b)
63+
Transformer
64+
fun redf b => redf
65+
[Meta.synthInstance] ✅️ apply @comp to ∀ (b : β), IsSmooth (f b)
66+
[Meta.synthInstance.tryResolve] ✅️ IsSmooth (f b) ≟ IsSmooth fun a => f b a
67+
[Meta.synthInstance] ❌️ apply @parm to ∀ (b : β), IsSmooth (f b)
68+
[Meta.synthInstance.tryResolve] ❌️ IsSmooth (f b) ≟ IsSmooth fun a => ?m b a (?m b)
69+
[Meta.synthInstance] ❌️ apply @const to ∀ (b : β), IsSmooth (f b)
70+
[Meta.synthInstance.tryResolve] ❌️ IsSmooth (f b) ≟ IsSmooth fun a => ?m b
71+
[Meta.synthInstance] ❌️ apply @identity to ∀ (b : β), IsSmooth (f b)
72+
[Meta.synthInstance.tryResolve] ❌️ IsSmooth (f b) ≟ IsSmooth fun a => a
5073
[Meta.synthInstance] ❌️ apply @comp to ∀ (a : α), IsSmooth fun g => f (g a) d
5174
[Meta.synthInstance.tryResolve] ❌️ IsSmooth fun g => f (g a) d ≟ IsSmooth fun a_1 => ?m a (?m a a_1)
5275
[Meta.synthInstance] ✅️ apply @parm to ∀ (a : α), IsSmooth fun g => f (g a) d
5376
[Meta.synthInstance.tryResolve] ✅️ IsSmooth fun g => f (g a) d ≟ IsSmooth fun a_1 => f (a_1 a) d
5477
[Meta.synthInstance] new goal ∀ (a : α), IsSmooth fun g => f (g a)
55-
[Meta.synthInstance.instances] #[@identity, @const, @parm, @comp, @diag, inst✝]
78+
[Meta.synthInstance.instances] #[@identity, @const, @parm, @comp, @diag, @swap, inst✝]
5679
[Meta.synthInstance] ❌️ apply inst✝ to ∀ (a : α), IsSmooth fun g => f (g a)
5780
[Meta.synthInstance.tryResolve] ❌️ IsSmooth fun g => f (g a) ≟ IsSmooth f
81+
[Meta.synthInstance] ✅️ apply @swap to ∀ (a : α), IsSmooth fun g => f (g a)
82+
[Meta.synthInstance.tryResolve] ✅️ IsSmooth fun g => f (g a) ≟ IsSmooth fun b a_1 => f (b a) a_1
83+
[Meta.synthInstance] new goal ∀ (a : α) (a_1 : δ), IsSmooth fun g => f (g a) a_1
84+
[Meta.synthInstance.instances] #[@identity, @const, @parm, @comp, @diag, inst✝]
85+
[Meta.synthInstance] ❌️ apply inst✝ to ∀ (a : α) (a_1 : δ), IsSmooth fun g => f (g a) a_1
86+
[Meta.synthInstance.tryResolve] ❌️ IsSmooth fun g => f (g a✝) a ≟ IsSmooth f
87+
[Meta.synthInstance] ✅️ apply @diag to ∀ (a : α) (a_1 : δ), IsSmooth fun g => f (g a) a_1
88+
[Meta.synthInstance.tryResolve] ✅️ IsSmooth fun g => f (g a✝) a ≟ IsSmooth fun a_1 => f (a_1 a✝) a
89+
[Meta.synthInstance.unusedArgs] ∀ (a : α) (a : δ), IsSmooth f
90+
has unused arguments, reduced type
91+
IsSmooth f
92+
Transformer
93+
fun redf a a => redf
94+
[Meta.synthInstance.resume] propagating ∀ (a : α) (a : δ),
95+
IsSmooth f to subgoal ∀ (a : α) (a : δ), IsSmooth f of ∀ (a : α) (a_1 : δ), IsSmooth fun g => f (g a) a_1
96+
[Meta.synthInstance.resume] size: 1
97+
[Meta.synthInstance.unusedArgs] ∀ (a : α) (a : δ) (b : β), IsSmooth (f b)
98+
has unused arguments, reduced type
99+
∀ (b : β), IsSmooth (f b)
100+
Transformer
101+
fun redf a a => redf
102+
[Meta.synthInstance] ❌️ apply @comp to ∀ (a : α) (a_1 : δ), IsSmooth fun g => f (g a) a_1
103+
[Meta.synthInstance.tryResolve] ❌️ IsSmooth fun g =>
104+
f (g a✝) a ≟ IsSmooth fun a_1 => ?m a✝ a (?m a✝ a a_1)
105+
[Meta.synthInstance] ✅️ apply @parm to ∀ (a : α) (a_1 : δ), IsSmooth fun g => f (g a) a_1
106+
[Meta.synthInstance.tryResolve] ✅️ IsSmooth fun g => f (g a✝) a ≟ IsSmooth fun a_1 => f (a_1 a✝) a
107+
[Meta.synthInstance.unusedArgs] ∀ (a : α) (a_1 : δ), IsSmooth fun g => f (g a)
108+
has unused arguments, reduced type
109+
∀ (a : α), IsSmooth fun g => f (g a)
110+
Transformer
111+
fun redf a a_1 => redf a
112+
[Meta.synthInstance] ❌️ apply @const to ∀ (a : α) (a_1 : δ), IsSmooth fun g => f (g a) a_1
113+
[Meta.synthInstance.tryResolve] ❌️ IsSmooth fun g => f (g a✝) a ≟ IsSmooth fun a_1 => ?m a✝ a
114+
[Meta.synthInstance] ❌️ apply @identity to ∀ (a : α) (a_1 : δ), IsSmooth fun g => f (g a) a_1
115+
[Meta.synthInstance.tryResolve] ❌️ IsSmooth fun g => f (g a✝) a ≟ IsSmooth fun a => a
58116
[Meta.synthInstance] ❌️ apply @diag to ∀ (a : α), IsSmooth fun g => f (g a)
59117
[Meta.synthInstance.tryResolve] ❌️ IsSmooth fun g =>
60118
f (g a) ≟ IsSmooth fun a_1 => ?m a (?m a a_1) (?m a a_1)

0 commit comments

Comments
 (0)