Register string positions with grind. #
Equations
- String.Internal.tacticOrder = Lean.ParserDescr.node `String.Internal.tacticOrder 1024 (Lean.ParserDescr.nonReservedSymbol "order" false)
Instances For
Equations
- String.Pos.Raw.instToIntCiOfNatInt = { toInt := fun (p : String.Pos.Raw) => ↑p.byteIdx, toInt_inj := ⋯, toInt_mem := String.Pos.Raw.instToIntCiOfNatInt._proof_4 }
instance
String.Pos.instToIntCoOfNatIntHAddCastUtf8ByteSize
{s : String}
:
Lean.Grind.ToInt s.Pos (Lean.Grind.IntInterval.co 0 (↑s.utf8ByteSize + 1))
instance
String.Pos.instLECoOfNatIntHAddCastUtf8ByteSize
{s : String}
:
Lean.Grind.ToInt.LE s.Pos (Lean.Grind.IntInterval.co 0 (↑s.utf8ByteSize + 1))
instance
String.Pos.instLTCoOfNatIntHAddCastUtf8ByteSize
{s : String}
:
Lean.Grind.ToInt.LT s.Pos (Lean.Grind.IntInterval.co 0 (↑s.utf8ByteSize + 1))
instance
String.Slice.Pos.instToIntCoOfNatIntHAddCastUtf8ByteSize
{s : Slice}
:
Lean.Grind.ToInt s.Pos (Lean.Grind.IntInterval.co 0 (↑s.utf8ByteSize + 1))
instance
String.Slice.Pos.instLECoOfNatIntHAddCastUtf8ByteSize
{s : Slice}
:
Lean.Grind.ToInt.LE s.Pos (Lean.Grind.IntInterval.co 0 (↑s.utf8ByteSize + 1))
instance
String.Slice.Pos.instLTCoOfNatIntHAddCastUtf8ByteSize
{s : Slice}
:
Lean.Grind.ToInt.LT s.Pos (Lean.Grind.IntInterval.co 0 (↑s.utf8ByteSize + 1))