Skip to content

Commit f73e69a

Browse files
committed
fix one test; the other can't be reproduced locally...
1 parent de78a66 commit f73e69a

File tree

1 file changed

+9
-6
lines changed

1 file changed

+9
-6
lines changed

tests/lean/binopInfoTree.lean.expected.out

Lines changed: 9 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -1,21 +1,21 @@
1-
[Elab.info]
1+
[Elab.info]
22
• [Command] @ ⟨3, 0⟩-⟨3, 31⟩ @ Lean.Elab.Command.elabSetOption
33
• [Completion] (Command.set_option "set_option" `trace.Elab.info []) @ ⟨3, 0⟩-⟨3, 26⟩
44
• [Option] trace.Elab.info @ ⟨3, 11⟩-⟨3, 26⟩
55
1 + 2 + 3 : Nat
6-
[Elab.info]
6+
[Elab.info]
77
• [Command] @ ⟨5, 0⟩-⟨5, 16⟩ @ Lean.Elab.Command.elabCheck
88
• [Term] 1 + 2 + 3 : Nat @ ⟨5, 7⟩-⟨5, 16⟩ @ «_aux_Init_Notation___macroRules_term_+__2»
99
• [MacroExpansion]
1010
1 + 2 +
1111
3
1212
-- should propagate through multiple macro expansions
13-
13+
1414
===>
1515
binop% HAdd.hAdd✝ (1 + 2)
1616
3
1717
-- should propagate through multiple macro expansions
18-
18+
1919
• [Term] 1 + 2 + 3 : Nat @ ⟨5, 7⟩†-⟨5, 16⟩† @ Lean.Elab.Term.Op.elabBinOp
2020
• [Term] 1 + 2 + 3 : Nat @ ⟨5, 7⟩†-⟨5, 16⟩†
2121
• [Term] 1 + 2 : Nat @ ⟨5, 7⟩-⟨5, 12⟩ @ «_aux_Init_Notation___macroRules_term_+__2»
@@ -30,7 +30,7 @@
3030
• [Term] 2 : Nat @ ⟨5, 11⟩-⟨5, 12⟩ @ Lean.Elab.Term.elabNumLit
3131
• [Term] 3 : Nat @ ⟨5, 15⟩-⟨5, 16⟩ @ Lean.Elab.Term.elabNumLit
3232
fun n m l => ↑n + (↑m + ↑l) : Nat → Nat → Nat → Int
33-
[Elab.info]
33+
[Elab.info]
3434
• [Command] @ ⟨7, 0⟩-⟨7, 48⟩ @ Lean.Elab.Command.elabCheck
3535
• [Term] fun n m l => ↑n + (↑m + ↑l) : Nat → Nat → Nat → Int @ ⟨7, 7⟩-⟨7, 48⟩ @ Lean.Elab.Term.elabFun
3636
• [Term] Nat : Type @ ⟨7, 20⟩-⟨7, 23⟩ @ Lean.Elab.Term.elabIdent
@@ -55,6 +55,9 @@ fun n m l => ↑n + (↑m + ↑l) : Nat → Nat → Nat → Int
5555
===>
5656
binop% HAdd.hAdd✝ n (m +' l)
5757
• [Term] ↑n + (↑m + ↑l) : Int @ ⟨7, 29⟩†-⟨7, 41⟩† @ Lean.Elab.Term.Op.elabBinOp
58+
• [CustomInfo(Lean.Elab.Term.CoeExpansionTrace)]
59+
• [CustomInfo(Lean.Elab.Term.CoeExpansionTrace)]
60+
• [CustomInfo(Lean.Elab.Term.CoeExpansionTrace)]
5861
• [Term] ↑n + (↑m + ↑l) : Int @ ⟨7, 29⟩†-⟨7, 41⟩†
5962
• [Completion-Id] HAdd.hAdd✝ : none @ ⟨7, 29⟩†-⟨7, 41⟩†
6063
• [Term] n : Nat @ ⟨7, 29⟩-⟨7, 30⟩ @ Lean.Elab.Term.elabIdent
@@ -78,5 +81,5 @@ fun n m l => ↑n + (↑m + ↑l) : Nat → Nat → Nat → Int
7881
• [Term] l : Nat @ ⟨7, 39⟩-⟨7, 40⟩ @ Lean.Elab.Term.elabIdent
7982
• [Completion-Id] l : none @ ⟨7, 39⟩-⟨7, 40⟩
8083
• [Term] l : Nat @ ⟨7, 39⟩-⟨7, 40⟩
81-
[Elab.info]
84+
[Elab.info]
8285
• [Command] @ ⟨8, 0⟩-⟨8, 0⟩ @ Lean.Elab.Command.elabEoi

0 commit comments

Comments
 (0)