author | wenzelm |
Tue, 12 Aug 2014 15:46:20 +0200 | |
changeset 57912 | dd9550f84106 |
parent 57620 | c30ab960875e |
child 58749 | 83b0f633190e |
permissions | -rw-r--r-- |
38425 | 1 |
/* Title: Pure/PIDE/text.scala |
45673
cd41e3903fbf
separate compilation of PIDE vs. Pure sources, which enables independent Scala library;
wenzelm
parents:
45667
diff
changeset
|
2 |
Module: PIDE |
34276 | 3 |
Author: Fabian Immler, TU Munich |
4 |
Author: Makarius |
|
5 |
||
38425 | 6 |
Basic operations on plain text. |
34276 | 7 |
*/ |
8 |
||
9 |
package isabelle |
|
10 |
||
11 |
||
44379 | 12 |
import scala.collection.mutable |
13 |
import scala.util.Sorting |
|
14 |
||
15 |
||
38425 | 16 |
object Text |
34276 | 17 |
{ |
38477 | 18 |
/* offset */ |
38426 | 19 |
|
20 |
type Offset = Int |
|
21 |
||
38477 | 22 |
|
38565
32b924a832c4
further clarification/unification of Position.Range and Text.Range concerning singularities: start offset is always included;
wenzelm
parents:
38564
diff
changeset
|
23 |
/* range -- with total quasi-ordering */ |
38477 | 24 |
|
38568 | 25 |
object Range |
26 |
{ |
|
27 |
def apply(start: Offset): Range = Range(start, start) |
|
44379 | 28 |
|
56172 | 29 |
val offside: Range = apply(-1) |
30 |
||
44379 | 31 |
object Ordering extends scala.math.Ordering[Text.Range] |
32 |
{ |
|
33 |
def compare(r1: Text.Range, r2: Text.Range): Int = r1 compare r2 |
|
34 |
} |
|
38568 | 35 |
} |
36 |
||
38426 | 37 |
sealed case class Range(val start: Offset, val stop: Offset) |
38427 | 38 |
{ |
38565
32b924a832c4
further clarification/unification of Position.Range and Text.Range concerning singularities: start offset is always included;
wenzelm
parents:
38564
diff
changeset
|
39 |
// denotation: {start} Un {i. start < i & i < stop} |
43425 | 40 |
if (start > stop) |
41 |
error("Bad range: [" + start.toString + ":" + stop.toString + "]") |
|
38477 | 42 |
|
57912 | 43 |
override def toString: String = "[" + start.toString + ":" + stop.toString + "]" |
38563 | 44 |
|
47542
26d0a76fef0a
more robust Sendback handling: JVM/jEdit paranoia for case matching, treat Pretty body not just XML.Text, replace proper_range only (without trailing whitespace);
wenzelm
parents:
46712
diff
changeset
|
45 |
def length: Int = stop - start |
26d0a76fef0a
more robust Sendback handling: JVM/jEdit paranoia for case matching, treat Pretty body not just XML.Text, replace proper_range only (without trailing whitespace);
wenzelm
parents:
46712
diff
changeset
|
46 |
|
38427 | 47 |
def map(f: Offset => Offset): Range = Range(f(start), f(stop)) |
56308 | 48 |
def +(i: Offset): Range = if (i == 0) this else map(_ + i) |
49 |
def -(i: Offset): Range = if (i == 0) this else map(_ - i) |
|
38662 | 50 |
|
38725 | 51 |
def is_singularity: Boolean = start == stop |
56590
d01d183e84ea
clarified treatment of markup ranges wrt. revert/convert: inflate_singularity allows to retrieve information like language_context more reliably during editing;
wenzelm
parents:
56473
diff
changeset
|
52 |
def inflate_singularity: Range = if (is_singularity) Range(start, start + 1) else this |
38662 | 53 |
|
38565
32b924a832c4
further clarification/unification of Position.Range and Text.Range concerning singularities: start offset is always included;
wenzelm
parents:
38564
diff
changeset
|
54 |
def contains(i: Offset): Boolean = start == i || start < i && i < stop |
32b924a832c4
further clarification/unification of Position.Range and Text.Range concerning singularities: start offset is always included;
wenzelm
parents:
38564
diff
changeset
|
55 |
def contains(that: Range): Boolean = this.contains(that.start) && that.stop <= this.stop |
32b924a832c4
further clarification/unification of Position.Range and Text.Range concerning singularities: start offset is always included;
wenzelm
parents:
38564
diff
changeset
|
56 |
def overlaps(that: Range): Boolean = this.contains(that.start) || that.contains(this.start) |
32b924a832c4
further clarification/unification of Position.Range and Text.Range concerning singularities: start offset is always included;
wenzelm
parents:
38564
diff
changeset
|
57 |
def compare(that: Range): Int = if (overlaps(that)) 0 else this.start compare that.start |
38485 | 58 |
|
45240
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
59 |
def apart(that: Range): Boolean = |
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
60 |
(this.start max that.start) > (this.stop min that.stop) |
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
61 |
|
38564 | 62 |
def restrict(that: Range): Range = |
38485 | 63 |
Range(this.start max that.start, this.stop min that.stop) |
43428
b41dea5772c6
more robust treatment of partial range restriction;
wenzelm
parents:
43425
diff
changeset
|
64 |
|
b41dea5772c6
more robust treatment of partial range restriction;
wenzelm
parents:
43425
diff
changeset
|
65 |
def try_restrict(that: Range): Option[Range] = |
45240
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
66 |
if (this apart that) None |
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
67 |
else Some(restrict(that)) |
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
68 |
|
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
69 |
def try_join(that: Range): Option[Range] = |
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
70 |
if (this apart that) None |
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
71 |
else Some(Range(this.start min that.start, this.stop max that.stop)) |
38427 | 72 |
} |
38426 | 73 |
|
74 |
||
44379 | 75 |
/* perspective */ |
76 |
||
44473 | 77 |
object Perspective |
44379 | 78 |
{ |
44474 | 79 |
val empty: Perspective = Perspective(Nil) |
44379 | 80 |
|
46576
ae9286f64574
approximate Perspective.full within the bounds of the JVM;
wenzelm
parents:
46207
diff
changeset
|
81 |
def full: Perspective = Perspective(List(Range(0, Integer.MAX_VALUE / 2))) |
ae9286f64574
approximate Perspective.full within the bounds of the JVM;
wenzelm
parents:
46207
diff
changeset
|
82 |
|
44473 | 83 |
def apply(ranges: Seq[Range]): Perspective = |
44379 | 84 |
{ |
44473 | 85 |
val result = new mutable.ListBuffer[Text.Range] |
86 |
var last: Option[Text.Range] = None |
|
45240
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
87 |
def ship(next: Option[Range]) { result ++= last; last = next } |
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
88 |
|
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
89 |
for (range <- ranges.sortBy(_.start)) |
44473 | 90 |
{ |
91 |
last match { |
|
45240
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
92 |
case None => ship(Some(range)) |
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
93 |
case Some(last_range) => |
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
94 |
last_range.try_join(range) match { |
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
95 |
case None => ship(Some(range)) |
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
96 |
case joined => last = joined |
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
97 |
} |
44473 | 98 |
} |
44379 | 99 |
} |
45240
9d97bd3c086a
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
wenzelm
parents:
44474
diff
changeset
|
100 |
ship(None) |
44473 | 101 |
new Perspective(result.toList) |
44379 | 102 |
} |
44473 | 103 |
} |
104 |
||
46712 | 105 |
final class Perspective private( |
106 |
val ranges: List[Range]) // visible text partitioning in canonical order |
|
44473 | 107 |
{ |
108 |
def is_empty: Boolean = ranges.isEmpty |
|
109 |
def range: Range = |
|
110 |
if (is_empty) Range(0) |
|
111 |
else Range(ranges.head.start, ranges.last.stop) |
|
45631
6bdf8b926f50
recovered structural equality from 9d97bd3c086a, otherwise update_perspective might be issued over and over again, canceling a pending/slow execution;
wenzelm
parents:
45470
diff
changeset
|
112 |
|
6bdf8b926f50
recovered structural equality from 9d97bd3c086a, otherwise update_perspective might be issued over and over again, canceling a pending/slow execution;
wenzelm
parents:
45470
diff
changeset
|
113 |
override def hashCode: Int = ranges.hashCode |
6bdf8b926f50
recovered structural equality from 9d97bd3c086a, otherwise update_perspective might be issued over and over again, canceling a pending/slow execution;
wenzelm
parents:
45470
diff
changeset
|
114 |
override def equals(that: Any): Boolean = |
6bdf8b926f50
recovered structural equality from 9d97bd3c086a, otherwise update_perspective might be issued over and over again, canceling a pending/slow execution;
wenzelm
parents:
45470
diff
changeset
|
115 |
that match { |
6bdf8b926f50
recovered structural equality from 9d97bd3c086a, otherwise update_perspective might be issued over and over again, canceling a pending/slow execution;
wenzelm
parents:
45470
diff
changeset
|
116 |
case other: Perspective => ranges == other.ranges |
6bdf8b926f50
recovered structural equality from 9d97bd3c086a, otherwise update_perspective might be issued over and over again, canceling a pending/slow execution;
wenzelm
parents:
45470
diff
changeset
|
117 |
case _ => false |
6bdf8b926f50
recovered structural equality from 9d97bd3c086a, otherwise update_perspective might be issued over and over again, canceling a pending/slow execution;
wenzelm
parents:
45470
diff
changeset
|
118 |
} |
57912 | 119 |
override def toString: String = ranges.toString |
44379 | 120 |
} |
121 |
||
122 |
||
38577 | 123 |
/* information associated with text range */ |
124 |
||
43714 | 125 |
sealed case class Info[A](val range: Text.Range, val info: A) |
38577 | 126 |
{ |
127 |
def restrict(r: Text.Range): Info[A] = Info(range.restrict(r), info) |
|
46207 | 128 |
def try_restrict(r: Text.Range): Option[Info[A]] = range.try_restrict(r).map(Info(_, info)) |
38577 | 129 |
} |
130 |
||
45470 | 131 |
type Markup = Info[XML.Elem] |
45455 | 132 |
|
38577 | 133 |
|
38426 | 134 |
/* editing */ |
34286 | 135 |
|
38425 | 136 |
object Edit |
137 |
{ |
|
38426 | 138 |
def insert(start: Offset, text: String): Edit = new Edit(true, start, text) |
139 |
def remove(start: Offset, text: String): Edit = new Edit(false, start, text) |
|
38425 | 140 |
} |
34286 | 141 |
|
46712 | 142 |
final class Edit private(val is_insert: Boolean, val start: Offset, val text: String) |
38425 | 143 |
{ |
57912 | 144 |
override def toString: String = |
38425 | 145 |
(if (is_insert) "Insert(" else "Remove(") + (start, text).toString + ")" |
34286 | 146 |
|
147 |
||
38425 | 148 |
/* transform offsets */ |
34286 | 149 |
|
38426 | 150 |
private def transform(do_insert: Boolean, i: Offset): Offset = |
151 |
if (i < start) i |
|
43425 | 152 |
else if (do_insert) i + text.length |
38426 | 153 |
else (i - text.length) max start |
34286 | 154 |
|
43425 | 155 |
def convert(i: Offset): Offset = transform(is_insert, i) |
156 |
def revert(i: Offset): Offset = transform(!is_insert, i) |
|
38425 | 157 |
|
34286 | 158 |
|
38425 | 159 |
/* edit strings */ |
160 |
||
38426 | 161 |
private def insert(i: Offset, string: String): String = |
162 |
string.substring(0, i) + text + string.substring(i) |
|
34276 | 163 |
|
38426 | 164 |
private def remove(i: Offset, count: Int, string: String): String = |
165 |
string.substring(0, i) + string.substring(i + count) |
|
38425 | 166 |
|
167 |
def can_edit(string: String, shift: Int): Boolean = |
|
168 |
shift <= start && start < shift + string.length |
|
169 |
||
170 |
def edit(string: String, shift: Int): (Option[Edit], String) = |
|
171 |
if (!can_edit(string, shift)) (Some(this), string) |
|
172 |
else if (is_insert) (None, insert(start - shift, string)) |
|
173 |
else { |
|
38426 | 174 |
val i = start - shift |
175 |
val count = text.length min (string.length - i) |
|
38425 | 176 |
val rest = |
177 |
if (count == text.length) None |
|
178 |
else Some(Edit.remove(start, text.substring(count))) |
|
38426 | 179 |
(rest, remove(i, count, string)) |
38425 | 180 |
} |
181 |
} |
|
34276 | 182 |
} |