@@ -34,20 +34,20 @@ fun n m l => ↑n + (↑m + ↑l) : Nat → Nat → Nat → Int
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.815 } @ ⟨7, 20⟩-⟨7, 23⟩
37+ • [Completion-Id] Nat : some Sort.{?_uniq} @ ⟨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.817 } @ ⟨7, 20⟩-⟨7, 23⟩
41+ • [Completion-Id] Nat : some Sort.{?_uniq} @ ⟨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.819 } @ ⟨7, 20⟩-⟨7, 23⟩
45+ • [Completion-Id] Nat : some Sort.{?_uniq} @ ⟨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.821 } @ ⟨7, 44⟩-⟨7, 47⟩
50+ • [Completion-Id] Int : some Sort.{?_uniq} @ ⟨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_binopInfoTree___macroRules_term_ +'__1»
66+ • [Term] ↑m + ↑l : Int @ ⟨7, 34⟩-⟨7, 40⟩ @ «_aux_lean_binopInfoTree___macroRules_term_ +'__1»
6767 • [MacroExpansion]
6868 m +' l
6969 ===>
0 commit comments