Skip to content

Commit 637e10e

Browse files
committed
really fix the binopInfoTree test
1 parent f73e69a commit 637e10e

File tree

1 file changed

+11
-11
lines changed

1 file changed

+11
-11
lines changed

tests/lean/binopInfoTree.lean.expected.out

Lines changed: 11 additions & 11 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,24 +30,24 @@
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
37-
• [Completion-Id] Nat : some Sort.{?_uniq} @ ⟨7, 20⟩-⟨7, 23⟩
37+
• [Completion-Id] Nat : some Sort.{?_uniq.815} @ ⟨7, 20⟩-⟨7, 23⟩
3838
• [Term] Nat : Type @ ⟨7, 20⟩-⟨7, 23⟩
3939
• [Term] n (isBinder := true) : Nat @ ⟨7, 12⟩-⟨7, 13⟩
4040
• [Term] Nat : Type @ ⟨7, 20⟩-⟨7, 23⟩ @ Lean.Elab.Term.elabIdent
41-
• [Completion-Id] Nat : some Sort.{?_uniq} @ ⟨7, 20⟩-⟨7, 23⟩
41+
• [Completion-Id] Nat : some Sort.{?_uniq.817} @ ⟨7, 20⟩-⟨7, 23⟩
4242
• [Term] Nat : Type @ ⟨7, 20⟩-⟨7, 23⟩
4343
• [Term] m (isBinder := true) : Nat @ ⟨7, 14⟩-⟨7, 15⟩
4444
• [Term] Nat : Type @ ⟨7, 20⟩-⟨7, 23⟩ @ Lean.Elab.Term.elabIdent
45-
• [Completion-Id] Nat : some Sort.{?_uniq} @ ⟨7, 20⟩-⟨7, 23⟩
45+
• [Completion-Id] Nat : some Sort.{?_uniq.819} @ ⟨7, 20⟩-⟨7, 23⟩
4646
• [Term] Nat : Type @ ⟨7, 20⟩-⟨7, 23⟩
4747
• [Term] l (isBinder := true) : Nat @ ⟨7, 16⟩-⟨7, 17⟩
4848
• [Term] ↑n + (↑m + ↑l) : Int @ ⟨7, 28⟩-⟨7, 48⟩ @ Lean.Elab.Term.elabTypeAscription
4949
• [Term] Int : Type @ ⟨7, 44⟩-⟨7, 47⟩ @ Lean.Elab.Term.elabIdent
50-
• [Completion-Id] Int : some Sort.{?_uniq} @ ⟨7, 44⟩-⟨7, 47⟩
50+
• [Completion-Id] Int : some Sort.{?_uniq.821} @ ⟨7, 44⟩-⟨7, 47⟩
5151
• [Term] Int : Type @ ⟨7, 44⟩-⟨7, 47⟩
5252
• [Term] ↑n + (↑m + ↑l) : Int @ ⟨7, 29⟩-⟨7, 41⟩ @ «_aux_Init_Notation___macroRules_term_+__2»
5353
• [MacroExpansion]
@@ -63,7 +63,7 @@ fun n m l => ↑n + (↑m + ↑l) : Nat → Nat → Nat → Int
6363
• [Term] n : Nat @ ⟨7, 29⟩-⟨7, 30⟩ @ Lean.Elab.Term.elabIdent
6464
• [Completion-Id] n : none @ ⟨7, 29⟩-⟨7, 30⟩
6565
• [Term] n : Nat @ ⟨7, 29⟩-⟨7, 30⟩
66-
• [Term] ↑m + ↑l : Int @ ⟨7, 34⟩-⟨7, 40⟩ @ «_aux_lean_binopInfoTree___macroRules_term_+'__1»
66+
• [Term] ↑m + ↑l : Int @ ⟨7, 34⟩-⟨7, 40⟩ @ «_aux_binopInfoTree___macroRules_term_+'__1»
6767
• [MacroExpansion]
6868
m +' l
6969
===>
@@ -81,5 +81,5 @@ fun n m l => ↑n + (↑m + ↑l) : Nat → Nat → Nat → Int
8181
• [Term] l : Nat @ ⟨7, 39⟩-⟨7, 40⟩ @ Lean.Elab.Term.elabIdent
8282
• [Completion-Id] l : none @ ⟨7, 39⟩-⟨7, 40⟩
8383
• [Term] l : Nat @ ⟨7, 39⟩-⟨7, 40⟩
84-
[Elab.info]
84+
[Elab.info]
8585
• [Command] @ ⟨8, 0⟩-⟨8, 0⟩ @ Lean.Elab.Command.elabEoi

0 commit comments

Comments
 (0)