src/Pure/General/symbol.scala
changeset 65196 e8760a98db78
parent 64682 7e119f32276a
child 65335 7634d33c1a79
--- a/src/Pure/General/symbol.scala	Sun Mar 12 13:48:10 2017 +0100
+++ b/src/Pure/General/symbol.scala	Sun Mar 12 14:23:38 2017 +0100
@@ -130,15 +130,6 @@
 
   def length(text: CharSequence): Int = iterator(text).length
 
-  object Length extends Text.Length
-  {
-    def apply(text: String): Int = length(text)
-    def offset(text: String, i: Int): Option[Text.Offset] =
-      if (i <= 0 || iterator(text).forall(s => s.length == 1)) Text.Length.offset(text, i)
-      else if (i <= length(text)) Some(iterator(text).take(i).mkString.length)
-      else None
-  }
-
 
   /* decoding offsets */