Documentation

Lean.Data.Position

structure Lean.Position:
Type
Equations
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
Equations
structure Lean.FileMap:
Type
Equations
class Lean.MonadFileMap (m : TypeType) :
Type
Instances
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.loop (pos : String.Pos) (str : String) (ps : Array String.Pos) (lines : Array Nat) (b : Nat) (e : Nat) :