Equations
- Lean.instInhabitedPosition = { default := { line := default, column := default } }
Equations
- Lean.instReprPosition = { reprPrec := [anonymous] }
Equations
- Lean.Position.lt _fun_discr _fun_discr = match _fun_discr, _fun_discr with | { line := l₁, column := c₁ }, { line := l₂, column := c₂ } => decide ((l₁, c₁) < (l₂, c₂))
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Position.instToExprPosition = { toExpr := fun p => Lean.mkAppN (Lean.mkConst `Lean.Position.mk) #[Lean.toExpr p.line, Lean.toExpr p.column], toTypeExpr := Lean.mkConst `Lean.Position }
Equations
- Lean.instInhabitedFileMap = { default := { source := default, positions := default, lines := default } }
- getFileMap : m Lean.FileMap
Instances
Equations
- Lean.FileMap.ofString s = Lean.FileMap.ofString.loop s 0 1 #[0] #[1]
partial def
Lean.FileMap.ofString.loop
(s : String)
(i : String.Pos)
(line : Nat)
(ps : Array String.Pos)
(lines : Array Nat)
:
Equations
- One or more equations did not get rendered due to their size.
partial def
Lean.FileMap.toPosition.toColumn
(pos : String.Pos)
(str : String)
(i : String.Pos)
(c : Nat)
:
partial def
Lean.FileMap.toPosition.loop
(pos : String.Pos)
(str : String)
(ps : Array String.Pos)
(lines : Array Nat)
(b : Nat)
(e : Nat)
: