| 518 |      1 | //Strong Bsimp to obtain Antimirov's cubic bound
 | 
|  |      2 | 
 | 
| 431 |      3 | // A simple lexer inspired by work of Sulzmann & Lu
 | 
|  |      4 | //==================================================
 | 
|  |      5 | //
 | 
|  |      6 | // Call the test cases with 
 | 
|  |      7 | //
 | 
|  |      8 | //   amm lexer.sc small
 | 
|  |      9 | //   amm lexer.sc fib
 | 
|  |     10 | //   amm lexer.sc loops
 | 
|  |     11 | //   amm lexer.sc email
 | 
|  |     12 | //
 | 
|  |     13 | //   amm lexer.sc all
 | 
|  |     14 | 
 | 
| 514 |     15 | 
 | 
| 431 |     16 | 
 | 
|  |     17 | // regular expressions including records
 | 
|  |     18 | abstract class Rexp 
 | 
|  |     19 | case object ZERO extends Rexp
 | 
|  |     20 | case object ONE extends Rexp
 | 
|  |     21 | case object ANYCHAR extends Rexp
 | 
|  |     22 | case class CHAR(c: Char) extends Rexp
 | 
|  |     23 | case class ALTS(r1: Rexp, r2: Rexp) extends Rexp 
 | 
|  |     24 | case class SEQ(r1: Rexp, r2: Rexp) extends Rexp 
 | 
|  |     25 | case class STAR(r: Rexp) extends Rexp 
 | 
|  |     26 | case class RECD(x: String, r: Rexp) extends Rexp  
 | 
|  |     27 | case class NTIMES(n: Int, r: Rexp) extends Rexp
 | 
|  |     28 | case class OPTIONAL(r: Rexp) extends Rexp
 | 
|  |     29 | case class NOT(r: Rexp) extends Rexp
 | 
|  |     30 |                 // records for extracting strings or tokens
 | 
|  |     31 |   
 | 
|  |     32 | // values  
 | 
|  |     33 | abstract class Val
 | 
| 492 |     34 | case object Failure extends Val
 | 
| 431 |     35 | case object Empty extends Val
 | 
|  |     36 | case class Chr(c: Char) extends Val
 | 
|  |     37 | case class Sequ(v1: Val, v2: Val) extends Val
 | 
|  |     38 | case class Left(v: Val) extends Val
 | 
|  |     39 | case class Right(v: Val) extends Val
 | 
|  |     40 | case class Stars(vs: List[Val]) extends Val
 | 
|  |     41 | case class Rec(x: String, v: Val) extends Val
 | 
|  |     42 | case class Ntime(vs: List[Val]) extends Val
 | 
|  |     43 | case class Optionall(v: Val) extends Val
 | 
|  |     44 | case class Nots(s: String) extends Val
 | 
|  |     45 | 
 | 
|  |     46 | 
 | 
|  |     47 | 
 | 
|  |     48 | abstract class Bit
 | 
|  |     49 | case object Z extends Bit
 | 
|  |     50 | case object S extends Bit
 | 
|  |     51 | 
 | 
|  |     52 | 
 | 
|  |     53 | type Bits = List[Bit]
 | 
|  |     54 | 
 | 
|  |     55 | abstract class ARexp 
 | 
|  |     56 | case object AZERO extends ARexp
 | 
|  |     57 | case class AONE(bs: Bits) extends ARexp
 | 
|  |     58 | case class ACHAR(bs: Bits, c: Char) extends ARexp
 | 
|  |     59 | case class AALTS(bs: Bits, rs: List[ARexp]) extends ARexp 
 | 
|  |     60 | case class ASEQ(bs: Bits, r1: ARexp, r2: ARexp) extends ARexp 
 | 
|  |     61 | case class ASTAR(bs: Bits, r: ARexp) extends ARexp 
 | 
|  |     62 | case class ANOT(bs: Bits, r: ARexp) extends ARexp
 | 
|  |     63 | case class AANYCHAR(bs: Bits) extends ARexp
 | 
|  |     64 | 
 | 
| 514 |     65 | import scala.util.Try
 | 
|  |     66 | 
 | 
| 492 |     67 | trait Generator[+T] {
 | 
|  |     68 |     self => // an alias for "this"
 | 
|  |     69 |     def generate(): T
 | 
|  |     70 |   
 | 
|  |     71 |     def gen(n: Int) : List[T] = 
 | 
|  |     72 |       if (n == 0) Nil else self.generate() :: gen(n - 1)
 | 
|  |     73 |     
 | 
|  |     74 |     def map[S](f: T => S): Generator[S] = new Generator[S] {
 | 
|  |     75 |       def generate = f(self.generate())  
 | 
|  |     76 |     }
 | 
|  |     77 |     def flatMap[S](f: T => Generator[S]): Generator[S] = new Generator[S] {
 | 
|  |     78 |       def generate = f(self.generate()).generate()
 | 
|  |     79 |     }
 | 
|  |     80 | 
 | 
|  |     81 | 
 | 
|  |     82 | }
 | 
|  |     83 | 
 | 
|  |     84 |   // tests a property according to a given random generator
 | 
|  |     85 |   def test[T](r: Generator[T], amount: Int = 100)(pred: T => Boolean) {
 | 
|  |     86 |     for (_ <- 0 until amount) {
 | 
|  |     87 |       val value = r.generate()
 | 
|  |     88 |       assert(pred(value), s"Test failed for: $value")
 | 
|  |     89 |     }
 | 
|  |     90 |     println(s"Test passed $amount times")
 | 
|  |     91 |   }
 | 
|  |     92 |   def test2[T, S](r: Generator[T], s: Generator[S], amount: Int = 100)(pred: (T, S) => Boolean) {
 | 
|  |     93 |     for (_ <- 0 until amount) {
 | 
|  |     94 |       val valueR = r.generate()
 | 
|  |     95 |       val valueS = s.generate()
 | 
|  |     96 |       assert(pred(valueR, valueS), s"Test failed for: $valueR, $valueS")
 | 
|  |     97 |     }
 | 
|  |     98 |     println(s"Test passed $amount times")
 | 
|  |     99 |   }
 | 
|  |    100 | 
 | 
|  |    101 | // random integers
 | 
|  |    102 | val integers = new Generator[Int] {
 | 
|  |    103 |   val rand = new java.util.Random
 | 
|  |    104 |   def generate() = rand.nextInt()
 | 
|  |    105 | }
 | 
|  |    106 | 
 | 
|  |    107 | // random booleans
 | 
|  |    108 | val booleans = integers.map(_ > 0)
 | 
|  |    109 |   
 | 
|  |    110 | // random integers in the range lo and high  
 | 
|  |    111 | def range(lo: Int, hi: Int): Generator[Int] = 
 | 
|  |    112 |   for (x <- integers) yield (lo + x.abs % (hi - lo)).abs
 | 
|  |    113 | 
 | 
|  |    114 | // random characters
 | 
|  |    115 | def chars_range(lo: Char, hi: Char) = range(lo, hi).map(_.toChar)  
 | 
|  |    116 | val chars = chars_range('a', 'z')
 | 
|  |    117 | 
 | 
|  |    118 | 
 | 
|  |    119 | def oneOf[T](xs: T*): Generator[T] = 
 | 
|  |    120 |   for (idx <- range(0, xs.length)) yield xs(idx)
 | 
|  |    121 |   
 | 
|  |    122 | def single[T](x: T) = new Generator[T] {
 | 
|  |    123 |   def generate() = x
 | 
|  |    124 | }   
 | 
|  |    125 | 
 | 
|  |    126 | def pairs[T, U](t: Generator[T], u: Generator[U]): Generator[(T, U)] = 
 | 
|  |    127 |   for (x <- t; y <- u) yield (x, y)
 | 
|  |    128 | 
 | 
|  |    129 | // lists
 | 
|  |    130 | def emptyLists = single(Nil) 
 | 
|  |    131 | 
 | 
|  |    132 | def nonEmptyLists : Generator[List[Int]] = 
 | 
|  |    133 |   for (head <- integers; tail <- lists) yield head :: tail
 | 
|  |    134 | 
 | 
|  |    135 | def lists: Generator[List[Int]] = for {
 | 
|  |    136 |   kind <- booleans
 | 
|  |    137 |   list <- if (kind) emptyLists else nonEmptyLists
 | 
|  |    138 | } yield list
 | 
|  |    139 | 
 | 
|  |    140 | def char_list(len: Int): Generator[List[Char]] = {
 | 
|  |    141 |   if(len <= 0) single(Nil)
 | 
|  |    142 |   else{
 | 
|  |    143 |     for { 
 | 
| 500 |    144 |       c <- chars_range('a', 'c')
 | 
| 492 |    145 |       tail <- char_list(len - 1)
 | 
|  |    146 |     } yield c :: tail
 | 
|  |    147 |   }
 | 
|  |    148 | }
 | 
|  |    149 | 
 | 
|  |    150 | def strings(len: Int): Generator[String] = for(cs <- char_list(len)) yield cs.toString
 | 
|  |    151 | 
 | 
| 493 |    152 | def sampleString(r: Rexp) : List[String] = r match {
 | 
|  |    153 |   case STAR(r) => stringsFromRexp(r).flatMap(s => List("", s, s ++ s))//only generate 0, 1, 2 reptitions
 | 
|  |    154 |   case SEQ(r1, r2) => stringsFromRexp(r1).flatMap(s1 => stringsFromRexp(r2).map(s2 => s1 ++ s2) )
 | 
|  |    155 |   case ALTS(r1, r2) => throw new Error(s" Rexp ${r} not expected: all alternatives are supposed to have been opened up")
 | 
|  |    156 |   case ONE => "" :: Nil
 | 
|  |    157 |   case ZERO => Nil
 | 
|  |    158 |   case CHAR(c) => c.toString :: Nil
 | 
|  |    159 | 
 | 
|  |    160 | }
 | 
|  |    161 | 
 | 
|  |    162 | def stringsFromRexp(r: Rexp) : List[String] = 
 | 
|  |    163 |   breakIntoTerms(r).flatMap(r => sampleString(r))
 | 
|  |    164 | 
 | 
| 492 |    165 | 
 | 
|  |    166 | // (simple) binary trees
 | 
|  |    167 | trait Tree[T]
 | 
|  |    168 | case class Inner[T](left: Tree[T], right: Tree[T]) extends Tree[T]
 | 
|  |    169 | case class Leaf[T](x: T) extends Tree[T]
 | 
|  |    170 | 
 | 
|  |    171 | def leafs[T](t: Generator[T]): Generator[Leaf[T]] = 
 | 
|  |    172 |   for (x <- t) yield Leaf(x)
 | 
|  |    173 | 
 | 
|  |    174 | def inners[T](t: Generator[T]): Generator[Inner[T]] = 
 | 
|  |    175 |   for (l <- trees(t); r <- trees(t)) yield Inner(l, r)
 | 
|  |    176 | 
 | 
|  |    177 | def trees[T](t: Generator[T]): Generator[Tree[T]] = 
 | 
|  |    178 |   for (kind <- range(0, 2);  
 | 
|  |    179 |        tree <- if (kind == 0) leafs(t) else inners(t)) yield tree
 | 
|  |    180 | 
 | 
|  |    181 | // regular expressions
 | 
|  |    182 | 
 | 
|  |    183 | // generates random leaf-regexes; prefers CHAR-regexes
 | 
|  |    184 | def leaf_rexp() : Generator[Rexp] =
 | 
|  |    185 |   for (kind <- range(0, 5);
 | 
|  |    186 |        c <- chars_range('a', 'd')) yield
 | 
|  |    187 |     kind match {
 | 
|  |    188 |       case 0 => ZERO
 | 
|  |    189 |       case 1 => ONE
 | 
|  |    190 |       case _ => CHAR(c) 
 | 
|  |    191 |     }
 | 
|  |    192 | 
 | 
|  |    193 | // generates random inner regexes with maximum depth d
 | 
|  |    194 | def inner_rexp(d: Int) : Generator[Rexp] =
 | 
|  |    195 |   for (kind <- range(0, 3);
 | 
|  |    196 |        l <- rexp(d); 
 | 
|  |    197 |        r <- rexp(d))
 | 
|  |    198 |   yield kind match {
 | 
|  |    199 |     case 0 => ALTS(l, r)
 | 
|  |    200 |     case 1 => SEQ(l, r)
 | 
|  |    201 |     case 2 => STAR(r)
 | 
|  |    202 |   }
 | 
|  |    203 | 
 | 
|  |    204 | // generates random regexes with maximum depth d;
 | 
|  |    205 | // prefers inner regexes in 2/3 of the cases
 | 
|  |    206 | def rexp(d: Int = 100): Generator[Rexp] = 
 | 
|  |    207 |   for (kind <- range(0, 3);
 | 
|  |    208 |        r <- if (d <= 0 || kind == 0) leaf_rexp() else inner_rexp(d - 1)) yield r
 | 
|  |    209 | 
 | 
|  |    210 | 
 | 
|  |    211 | // some test functions for rexps
 | 
|  |    212 | def height(r: Rexp) : Int = r match {
 | 
|  |    213 |   case ZERO => 1
 | 
|  |    214 |   case ONE => 1
 | 
|  |    215 |   case CHAR(_) => 1
 | 
|  |    216 |   case ALTS(r1, r2) => 1 + List(height(r1), height(r2)).max
 | 
|  |    217 |   case SEQ(r1, r2) =>  1 + List(height(r1), height(r2)).max
 | 
|  |    218 |   case STAR(r) => 1 + height(r)
 | 
|  |    219 | }
 | 
|  |    220 | 
 | 
|  |    221 | // def size(r: Rexp) : Int = r match {
 | 
|  |    222 | //   case ZERO => 1
 | 
|  |    223 | //   case ONE => 1
 | 
|  |    224 | //   case CHAR(_) => 1
 | 
|  |    225 | //   case ALTS(r1, r2) => 1 + size(r1) + size(r2)
 | 
|  |    226 | //   case SEQ(r1, r2) =>  1 + size(r1) + size(r2)
 | 
|  |    227 | //   case STAR(r) => 1 + size(r) 
 | 
|  |    228 | // }
 | 
|  |    229 | 
 | 
|  |    230 | // randomly subtracts 1 or 2 from the STAR case
 | 
|  |    231 | def size_faulty(r: Rexp) : Int = r match {
 | 
|  |    232 |   case ZERO => 1
 | 
|  |    233 |   case ONE => 1
 | 
|  |    234 |   case CHAR(_) => 1
 | 
|  |    235 |   case ALTS(r1, r2) => 1 + size_faulty(r1) + size_faulty(r2)
 | 
|  |    236 |   case SEQ(r1, r2) =>  1 + size_faulty(r1) + size_faulty(r2)
 | 
|  |    237 |   case STAR(r) => 1 + size_faulty(r) - range(0, 2).generate
 | 
|  |    238 | }
 | 
|  |    239 | 
 | 
| 431 |    240 | 
 | 
|  |    241 |    
 | 
|  |    242 | // some convenience for typing in regular expressions
 | 
|  |    243 | 
 | 
|  |    244 | def charlist2rexp(s : List[Char]): Rexp = s match {
 | 
|  |    245 |   case Nil => ONE
 | 
|  |    246 |   case c::Nil => CHAR(c)
 | 
|  |    247 |   case c::s => SEQ(CHAR(c), charlist2rexp(s))
 | 
|  |    248 | }
 | 
|  |    249 | implicit def string2rexp(s : String) : Rexp = 
 | 
|  |    250 |   charlist2rexp(s.toList)
 | 
|  |    251 | 
 | 
|  |    252 | implicit def RexpOps(r: Rexp) = new {
 | 
|  |    253 |   def | (s: Rexp) = ALTS(r, s)
 | 
|  |    254 |   def % = STAR(r)
 | 
|  |    255 |   def ~ (s: Rexp) = SEQ(r, s)
 | 
|  |    256 | }
 | 
|  |    257 | 
 | 
|  |    258 | implicit def stringOps(s: String) = new {
 | 
|  |    259 |   def | (r: Rexp) = ALTS(s, r)
 | 
|  |    260 |   def | (r: String) = ALTS(s, r)
 | 
|  |    261 |   def % = STAR(s)
 | 
|  |    262 |   def ~ (r: Rexp) = SEQ(s, r)
 | 
|  |    263 |   def ~ (r: String) = SEQ(s, r)
 | 
|  |    264 |   def $ (r: Rexp) = RECD(s, r)
 | 
|  |    265 | }
 | 
|  |    266 | 
 | 
|  |    267 | def nullable(r: Rexp) : Boolean = r match {
 | 
|  |    268 |   case ZERO => false
 | 
|  |    269 |   case ONE => true
 | 
|  |    270 |   case CHAR(_) => false
 | 
|  |    271 |   case ANYCHAR => false
 | 
|  |    272 |   case ALTS(r1, r2) => nullable(r1) || nullable(r2)
 | 
|  |    273 |   case SEQ(r1, r2) => nullable(r1) && nullable(r2)
 | 
|  |    274 |   case STAR(_) => true
 | 
|  |    275 |   case RECD(_, r1) => nullable(r1)
 | 
|  |    276 |   case NTIMES(n, r) => if (n == 0) true else nullable(r)
 | 
|  |    277 |   case OPTIONAL(r) => true
 | 
|  |    278 |   case NOT(r) => !nullable(r)
 | 
|  |    279 | }
 | 
|  |    280 | 
 | 
|  |    281 | def der(c: Char, r: Rexp) : Rexp = r match {
 | 
|  |    282 |   case ZERO => ZERO
 | 
|  |    283 |   case ONE => ZERO
 | 
|  |    284 |   case CHAR(d) => if (c == d) ONE else ZERO
 | 
|  |    285 |   case ANYCHAR => ONE 
 | 
|  |    286 |   case ALTS(r1, r2) => ALTS(der(c, r1), der(c, r2))
 | 
|  |    287 |   case SEQ(r1, r2) => 
 | 
|  |    288 |     if (nullable(r1)) ALTS(SEQ(der(c, r1), r2), der(c, r2))
 | 
|  |    289 |     else SEQ(der(c, r1), r2)
 | 
|  |    290 |   case STAR(r) => SEQ(der(c, r), STAR(r))
 | 
|  |    291 |   case RECD(_, r1) => der(c, r1)
 | 
|  |    292 |   case NTIMES(n, r) => if(n > 0) SEQ(der(c, r), NTIMES(n - 1, r)) else ZERO
 | 
|  |    293 |   case OPTIONAL(r) => der(c, r)
 | 
|  |    294 |   case NOT(r) =>  NOT(der(c, r))
 | 
|  |    295 | }
 | 
|  |    296 | 
 | 
|  |    297 | 
 | 
|  |    298 | // extracts a string from a value
 | 
|  |    299 | def flatten(v: Val) : String = v match {
 | 
|  |    300 |   case Empty => ""
 | 
|  |    301 |   case Chr(c) => c.toString
 | 
|  |    302 |   case Left(v) => flatten(v)
 | 
|  |    303 |   case Right(v) => flatten(v)
 | 
|  |    304 |   case Sequ(v1, v2) => flatten(v1) ++ flatten(v2)
 | 
|  |    305 |   case Stars(vs) => vs.map(flatten).mkString
 | 
|  |    306 |   case Ntime(vs) => vs.map(flatten).mkString
 | 
|  |    307 |   case Optionall(v) => flatten(v)
 | 
|  |    308 |   case Rec(_, v) => flatten(v)
 | 
|  |    309 | }
 | 
|  |    310 | 
 | 
|  |    311 | 
 | 
|  |    312 | // extracts an environment from a value;
 | 
|  |    313 | // used for tokenising a string
 | 
|  |    314 | def env(v: Val) : List[(String, String)] = v match {
 | 
|  |    315 |   case Empty => Nil
 | 
|  |    316 |   case Chr(c) => Nil
 | 
|  |    317 |   case Left(v) => env(v)
 | 
|  |    318 |   case Right(v) => env(v)
 | 
|  |    319 |   case Sequ(v1, v2) => env(v1) ::: env(v2)
 | 
|  |    320 |   case Stars(vs) => vs.flatMap(env)
 | 
|  |    321 |   case Ntime(vs) => vs.flatMap(env)
 | 
|  |    322 |   case Rec(x, v) => (x, flatten(v))::env(v)
 | 
|  |    323 |   case Optionall(v) => env(v)
 | 
|  |    324 |   case Nots(s) => ("Negative", s) :: Nil
 | 
|  |    325 | }
 | 
|  |    326 | 
 | 
|  |    327 | 
 | 
|  |    328 | // The injection and mkeps part of the lexer
 | 
|  |    329 | //===========================================
 | 
|  |    330 | 
 | 
|  |    331 | def mkeps(r: Rexp) : Val = r match {
 | 
|  |    332 |   case ONE => Empty
 | 
|  |    333 |   case ALTS(r1, r2) => 
 | 
|  |    334 |     if (nullable(r1)) Left(mkeps(r1)) else Right(mkeps(r2))
 | 
|  |    335 |   case SEQ(r1, r2) => Sequ(mkeps(r1), mkeps(r2))
 | 
|  |    336 |   case STAR(r) => Stars(Nil)
 | 
|  |    337 |   case RECD(x, r) => Rec(x, mkeps(r))
 | 
|  |    338 |   case NTIMES(n, r) => Ntime(List.fill(n)(mkeps(r)))
 | 
|  |    339 |   case OPTIONAL(r) => Optionall(Empty)
 | 
|  |    340 |   case NOT(rInner) => if(nullable(rInner)) throw new Exception("error")  
 | 
|  |    341 |                          else Nots("")//Nots(s.reverse.toString)
 | 
|  |    342 | //   case NOT(ZERO) => Empty
 | 
|  |    343 | //   case NOT(CHAR(c)) => Empty
 | 
|  |    344 | //   case NOT(SEQ(r1, r2)) => Sequ(mkeps(NOT(r1)), mkeps(NOT(r2)))
 | 
|  |    345 | //   case NOT(ALTS(r1, r2)) => if(!nullable(r1)) Left(mkeps(NOT(r1))) else Right(mkeps(NOT(r2)))
 | 
|  |    346 | //   case NOT(STAR(r)) => Stars(Nil) 
 | 
|  |    347 | 
 | 
|  |    348 | }
 | 
|  |    349 | 
 | 
|  |    350 | def inj(r: Rexp, c: Char, v: Val) : Val = (r, v) match {
 | 
|  |    351 |   case (STAR(r), Sequ(v1, Stars(vs))) => Stars(inj(r, c, v1)::vs)
 | 
|  |    352 |   case (SEQ(r1, r2), Sequ(v1, v2)) => Sequ(inj(r1, c, v1), v2)
 | 
|  |    353 |   case (SEQ(r1, r2), Left(Sequ(v1, v2))) => Sequ(inj(r1, c, v1), v2)
 | 
|  |    354 |   case (SEQ(r1, r2), Right(v2)) => Sequ(mkeps(r1), inj(r2, c, v2))
 | 
|  |    355 |   case (ALTS(r1, r2), Left(v1)) => Left(inj(r1, c, v1))
 | 
|  |    356 |   case (ALTS(r1, r2), Right(v2)) => Right(inj(r2, c, v2))
 | 
|  |    357 |   case (CHAR(d), Empty) => Chr(c) 
 | 
|  |    358 |   case (RECD(x, r1), _) => Rec(x, inj(r1, c, v))
 | 
|  |    359 |   case (NTIMES(n, r), Sequ(v1, Ntime(vs))) => Ntime(inj(r, c, v1)::vs)
 | 
|  |    360 |   case (OPTIONAL(r), v) => Optionall(inj(r, c, v))
 | 
|  |    361 |   case (NOT(r), Nots(s)) => Nots(c.toString ++ s)
 | 
|  |    362 |   case (ANYCHAR, Empty) => Chr(c)
 | 
|  |    363 | }
 | 
|  |    364 | 
 | 
|  |    365 | // some "rectification" functions for simplification
 | 
|  |    366 | 
 | 
|  |    367 | 
 | 
|  |    368 | 
 | 
|  |    369 | 
 | 
|  |    370 | // The Lexing Rules for the WHILE Language
 | 
|  |    371 | 
 | 
|  |    372 |   // bnullable function: tests whether the aregular 
 | 
|  |    373 |   // expression can recognise the empty string
 | 
|  |    374 | def bnullable (r: ARexp) : Boolean = r match {
 | 
|  |    375 |     case AZERO => false
 | 
|  |    376 |     case AONE(_) => true
 | 
|  |    377 |     case ACHAR(_,_) => false
 | 
|  |    378 |     case AALTS(_, rs) => rs.exists(bnullable)
 | 
|  |    379 |     case ASEQ(_, r1, r2) => bnullable(r1) && bnullable(r2)
 | 
|  |    380 |     case ASTAR(_, _) => true
 | 
|  |    381 |     case ANOT(_, rn) => !bnullable(rn)
 | 
|  |    382 |   }
 | 
|  |    383 | 
 | 
|  |    384 | def mkepsBC(r: ARexp) : Bits = r match {
 | 
|  |    385 |     case AONE(bs) => bs
 | 
|  |    386 |     case AALTS(bs, rs) => {
 | 
|  |    387 |       val n = rs.indexWhere(bnullable)
 | 
|  |    388 |       bs ++ mkepsBC(rs(n))
 | 
|  |    389 |     }
 | 
|  |    390 |     case ASEQ(bs, r1, r2) => bs ++ mkepsBC(r1) ++ mkepsBC(r2)
 | 
|  |    391 |     case ASTAR(bs, r) => bs ++ List(Z)
 | 
|  |    392 |     case ANOT(bs, rn) => bs
 | 
|  |    393 |   }
 | 
|  |    394 | 
 | 
|  |    395 | 
 | 
|  |    396 | def bder(c: Char, r: ARexp) : ARexp = r match {
 | 
|  |    397 |     case AZERO => AZERO
 | 
|  |    398 |     case AONE(_) => AZERO
 | 
|  |    399 |     case ACHAR(bs, f) => if (c == f) AONE(bs) else AZERO
 | 
|  |    400 |     case AALTS(bs, rs) => AALTS(bs, rs.map(bder(c, _)))
 | 
|  |    401 |     case ASEQ(bs, r1, r2) => 
 | 
|  |    402 |       if (bnullable(r1)) AALTS(bs, ASEQ(Nil, bder(c, r1), r2) :: fuse(mkepsBC(r1), bder(c, r2)) :: Nil )
 | 
|  |    403 |       else ASEQ(bs, bder(c, r1), r2)
 | 
|  |    404 |     case ASTAR(bs, r) => ASEQ(bs, fuse(List(S), bder(c, r)), ASTAR(Nil, r))
 | 
|  |    405 |     case ANOT(bs, rn) => ANOT(bs, bder(c, rn))
 | 
|  |    406 |     case AANYCHAR(bs) => AONE(bs)
 | 
|  |    407 |   } 
 | 
|  |    408 | 
 | 
|  |    409 | def fuse(bs: Bits, r: ARexp) : ARexp = r match {
 | 
|  |    410 |     case AZERO => AZERO
 | 
|  |    411 |     case AONE(cs) => AONE(bs ++ cs)
 | 
|  |    412 |     case ACHAR(cs, f) => ACHAR(bs ++ cs, f)
 | 
|  |    413 |     case AALTS(cs, rs) => AALTS(bs ++ cs, rs)
 | 
|  |    414 |     case ASEQ(cs, r1, r2) => ASEQ(bs ++ cs, r1, r2)
 | 
|  |    415 |     case ASTAR(cs, r) => ASTAR(bs ++ cs, r)
 | 
|  |    416 |     case ANOT(cs, r) => ANOT(bs ++ cs, r)
 | 
|  |    417 |   }
 | 
|  |    418 | 
 | 
|  |    419 | 
 | 
|  |    420 | def internalise(r: Rexp) : ARexp = r match {
 | 
|  |    421 |     case ZERO => AZERO
 | 
|  |    422 |     case ONE => AONE(Nil)
 | 
|  |    423 |     case CHAR(c) => ACHAR(Nil, c)
 | 
|  |    424 |     //case PRED(f) => APRED(Nil, f)
 | 
|  |    425 |     case ALTS(r1, r2) => 
 | 
|  |    426 |       AALTS(Nil, List(fuse(List(Z), internalise(r1)), fuse(List(S), internalise(r2))))
 | 
|  |    427 |     // case ALTS(r1::rs) => {
 | 
|  |    428 |     //   val AALTS(Nil, rs2) = internalise(ALTS(rs))
 | 
|  |    429 |     //   AALTS(Nil, fuse(List(Z), internalise(r1)) :: rs2.map(fuse(List(S), _)))
 | 
|  |    430 |     // }
 | 
|  |    431 |     case SEQ(r1, r2) => ASEQ(Nil, internalise(r1), internalise(r2))
 | 
|  |    432 |     case STAR(r) => ASTAR(Nil, internalise(r))
 | 
|  |    433 |     case RECD(x, r) => internalise(r)
 | 
|  |    434 |     case NOT(r) => ANOT(Nil, internalise(r))
 | 
|  |    435 |     case ANYCHAR => AANYCHAR(Nil)
 | 
|  |    436 |   }
 | 
|  |    437 | 
 | 
|  |    438 | 
 | 
|  |    439 | def bsimp(r: ARexp): ARexp = 
 | 
|  |    440 |   {
 | 
|  |    441 |     r match {
 | 
|  |    442 |       case ASEQ(bs1, r1, r2) => (bsimp(r1), bsimp(r2)) match {
 | 
|  |    443 |           case (AZERO, _) => AZERO
 | 
|  |    444 |           case (_, AZERO) => AZERO
 | 
|  |    445 |           case (AONE(bs2), r2s) => fuse(bs1 ++ bs2, r2s)
 | 
|  |    446 |           case (r1s, r2s) => ASEQ(bs1, r1s, r2s)
 | 
|  |    447 |       }
 | 
|  |    448 |       case AALTS(bs1, rs) => {
 | 
|  |    449 |             val rs_simp = rs.map(bsimp(_))
 | 
|  |    450 |             val flat_res = flats(rs_simp)
 | 
|  |    451 |             val dist_res = distinctBy(flat_res, erase)//strongDB(flat_res)//distinctBy(flat_res, erase)
 | 
|  |    452 |             dist_res match {
 | 
|  |    453 |               case Nil => AZERO
 | 
|  |    454 |               case s :: Nil => fuse(bs1, s)
 | 
|  |    455 |               case rs => AALTS(bs1, rs)  
 | 
|  |    456 |             }
 | 
|  |    457 |           
 | 
|  |    458 |       }
 | 
|  |    459 |       case r => r
 | 
|  |    460 |     }
 | 
| 492 |    461 | }
 | 
|  |    462 | def strongBsimp(r: ARexp): ARexp =
 | 
|  |    463 | {
 | 
|  |    464 |   r match {
 | 
|  |    465 |     case ASEQ(bs1, r1, r2) => (strongBsimp(r1), strongBsimp(r2)) match {
 | 
|  |    466 |         case (AZERO, _) => AZERO
 | 
|  |    467 |         case (_, AZERO) => AZERO
 | 
|  |    468 |         case (AONE(bs2), r2s) => fuse(bs1 ++ bs2, r2s)
 | 
|  |    469 |         case (r1s, r2s) => ASEQ(bs1, r1s, r2s)
 | 
| 431 |    470 |     }
 | 
| 492 |    471 |     case AALTS(bs1, rs) => {
 | 
|  |    472 |           val rs_simp = rs.map(strongBsimp(_))
 | 
|  |    473 |           val flat_res = flats(rs_simp)
 | 
|  |    474 |           val dist_res = distinctBy4(flat_res)//distinctBy(flat_res, erase)
 | 
|  |    475 |           dist_res match {
 | 
|  |    476 |             case Nil => AZERO
 | 
|  |    477 |             case s :: Nil => fuse(bs1, s)
 | 
|  |    478 |             case rs => AALTS(bs1, rs)  
 | 
|  |    479 |           }
 | 
|  |    480 |         
 | 
|  |    481 |     }
 | 
|  |    482 |     case r => r
 | 
| 431 |    483 |   }
 | 
| 492 |    484 | }
 | 
| 431 |    485 | 
 | 
| 494 |    486 | def strongBsimp5(r: ARexp): ARexp =
 | 
|  |    487 | {
 | 
|  |    488 |   // println("was this called?")
 | 
|  |    489 |   r match {
 | 
|  |    490 |     case ASEQ(bs1, r1, r2) => (strongBsimp5(r1), strongBsimp5(r2)) match {
 | 
|  |    491 |         case (AZERO, _) => AZERO
 | 
|  |    492 |         case (_, AZERO) => AZERO
 | 
|  |    493 |         case (AONE(bs2), r2s) => fuse(bs1 ++ bs2, r2s)
 | 
|  |    494 |         case (r1s, r2s) => ASEQ(bs1, r1s, r2s)
 | 
|  |    495 |     }
 | 
|  |    496 |     case AALTS(bs1, rs) => {
 | 
|  |    497 |         // println("alts case")
 | 
|  |    498 |           val rs_simp = rs.map(strongBsimp5(_))
 | 
|  |    499 |           val flat_res = flats(rs_simp)
 | 
| 500 |    500 |           var dist_res = distinctBy5(flat_res)//distinctBy(flat_res, erase)
 | 
| 518 |    501 |           // var dist2_res = distinctBy5(dist_res)
 | 
|  |    502 |           // while(dist_res != dist2_res){
 | 
|  |    503 |           //   dist_res = dist2_res
 | 
|  |    504 |           //   dist2_res = distinctBy5(dist_res)
 | 
|  |    505 |           // }
 | 
|  |    506 |           (dist_res) match {
 | 
|  |    507 |             case Nil => AZERO
 | 
|  |    508 |             case s :: Nil => fuse(bs1, s)
 | 
|  |    509 |             case rs => AALTS(bs1, rs)  
 | 
| 500 |    510 |           }
 | 
| 518 |    511 |     }
 | 
|  |    512 |     case r => r
 | 
|  |    513 |   }
 | 
|  |    514 | }
 | 
|  |    515 | 
 | 
|  |    516 | def strongBsimp6(r: ARexp): ARexp =
 | 
|  |    517 | {
 | 
|  |    518 |   // println("was this called?")
 | 
|  |    519 |   r match {
 | 
|  |    520 |     case ASEQ(bs1, r1, r2) => (strongBsimp6(r1), strongBsimp6(r2)) match {
 | 
|  |    521 |         case (AZERO, _) => AZERO
 | 
|  |    522 |         case (_, AZERO) => AZERO
 | 
|  |    523 |         case (AONE(bs2), r2s) => fuse(bs1 ++ bs2, r2s)
 | 
| 530 |    524 |         case (r1s, AONE(bs2)) => fuse(bs1, r1s) //asserted bs2 == Nil
 | 
| 532 |    525 |         //case (r1s, r2s) if(isOne(erase(r1s))) => fuse(bs1 ++ mkepsBC(r1s), r2s)
 | 
| 518 |    526 |         case (r1s, r2s) => ASEQ(bs1, r1s, r2s)
 | 
|  |    527 |     }
 | 
|  |    528 |     case AALTS(bs1, rs) => {
 | 
|  |    529 |         // println("alts case")
 | 
|  |    530 |           val rs_simp = rs.map(strongBsimp6(_))
 | 
|  |    531 |           val flat_res = flats(rs_simp)
 | 
|  |    532 |           var dist_res = distinctBy6(flat_res)//distinctBy(flat_res, erase)
 | 
|  |    533 |           (dist_res) match {
 | 
| 494 |    534 |             case Nil => AZERO
 | 
|  |    535 |             case s :: Nil => fuse(bs1, s)
 | 
|  |    536 |             case rs => AALTS(bs1, rs)  
 | 
|  |    537 |           }
 | 
|  |    538 |     }
 | 
| 532 |    539 |     case ASTAR(bs, r0) if(atMostEmpty(erase(r0))) => AONE(bs)
 | 
| 494 |    540 |     case r => r
 | 
|  |    541 |   }
 | 
|  |    542 | }
 | 
|  |    543 | 
 | 
| 532 |    544 | def distinctWith(rs: List[ARexp], 
 | 
|  |    545 |                 f: (ARexp, Set[Rexp]) => ARexp, 
 | 
|  |    546 |                 acc: Set[Rexp] = Set()) : List[ARexp] = 
 | 
|  |    547 |   rs match{
 | 
|  |    548 |     case Nil => Nil
 | 
|  |    549 |     case r :: rs => 
 | 
|  |    550 |       if(acc(erase(r)))
 | 
|  |    551 |         distinctWith(rs, f, acc)
 | 
|  |    552 |       else {
 | 
|  |    553 |         val pruned_r = f(r, acc)
 | 
|  |    554 |         pruned_r :: distinctWith(rs, f, strongBreakIntoTerms(erase(pruned_r)) ++: acc)
 | 
|  |    555 |       }
 | 
|  |    556 |   }
 | 
|  |    557 | 
 | 
|  |    558 | //r = r' ~ tail => returns r'
 | 
|  |    559 | def removeSeqTail(r: Rexp, tail: Rexp) : Rexp = r match {
 | 
|  |    560 |   case SEQ(r1, r2) => 
 | 
|  |    561 |     if(r2 == tail) 
 | 
|  |    562 |       r1
 | 
|  |    563 |     else
 | 
|  |    564 |       ZERO
 | 
|  |    565 |   case r => ZERO
 | 
|  |    566 | }
 | 
|  |    567 | 
 | 
|  |    568 | def prune7(r: ARexp, acc: Set[Rexp]) : ARexp = r match{
 | 
|  |    569 |   case AALTS(bs, rs) => rs.map(r => prune7(r, acc)).filter(_ != ZERO) match
 | 
|  |    570 |   {
 | 
|  |    571 |     case Nil => AZERO
 | 
|  |    572 |     case r::Nil => fuse(bs, r)
 | 
|  |    573 |     case rs1 => AALTS(bs, rs1)
 | 
|  |    574 |   }
 | 
|  |    575 |   case ASEQ(bs, r1, r2) => prune7(r1, acc.map(r => removeSeqTail(r, erase(r2)))) match {
 | 
|  |    576 |     case AZERO => AZERO
 | 
|  |    577 |     case r1p if(isOne(erase(r1p))) => fuse(bs ++ mkepsBC(r1p), r2)
 | 
|  |    578 |     case r1p => ASEQ(bs, r1p, r2)
 | 
|  |    579 |   }
 | 
|  |    580 |   case r => if(acc(erase(r))) AZERO else r
 | 
|  |    581 | }
 | 
|  |    582 | 
 | 
|  |    583 | def strongBsimp7(r: ARexp): ARexp =
 | 
|  |    584 | {
 | 
|  |    585 |   r match {
 | 
|  |    586 |     case ASEQ(bs1, r1, r2) => (strongBsimp7(r1), strongBsimp7(r2)) match {
 | 
|  |    587 |         case (AZERO, _) => AZERO
 | 
|  |    588 |         case (_, AZERO) => AZERO
 | 
|  |    589 |         case (AONE(bs2), r2s) => fuse(bs1 ++ bs2, r2s)
 | 
|  |    590 |         case (r1s, AONE(bs2)) => fuse(bs1, r1s) //asserted bs2 == Nil
 | 
|  |    591 |         //case (r1s, r2s) if(isOne(erase(r1s))) => fuse(bs1 ++ mkepsBC(r1s), r2s)
 | 
|  |    592 |         case (r1s, r2s) => ASEQ(bs1, r1s, r2s)
 | 
|  |    593 |     }
 | 
|  |    594 |     case AALTS(bs1, rs) => {
 | 
|  |    595 |         // println("alts case")
 | 
|  |    596 |           val rs_simp = rs.map(strongBsimp7(_))
 | 
|  |    597 |           val flat_res = flats(rs_simp)
 | 
|  |    598 |           var dist_res = distinctWith(flat_res, prune7)//distinctBy(flat_res, erase)
 | 
|  |    599 |           (dist_res) match {
 | 
|  |    600 |             case Nil => AZERO
 | 
|  |    601 |             case s :: Nil => fuse(bs1, s)
 | 
|  |    602 |             case rs => AALTS(bs1, rs)  
 | 
|  |    603 |           }
 | 
|  |    604 |     }
 | 
|  |    605 |     case ASTAR(bs, r0) if(atMostEmpty(erase(r0))) => AONE(bs)
 | 
|  |    606 |     case r => r
 | 
|  |    607 |   }
 | 
|  |    608 | }
 | 
|  |    609 | 
 | 
|  |    610 | 
 | 
| 492 |    611 | def bders (s: List[Char], r: ARexp) : ARexp = s match {
 | 
|  |    612 |   case Nil => r
 | 
|  |    613 |   case c::s => bders(s, bder(c, r))
 | 
|  |    614 | }
 | 
| 431 |    615 | 
 | 
| 492 |    616 | def flats(rs: List[ARexp]): List[ARexp] = rs match {
 | 
| 431 |    617 |     case Nil => Nil
 | 
| 492 |    618 |     case AZERO :: rs1 => flats(rs1)
 | 
|  |    619 |     case AALTS(bs, rs1) :: rs2 => rs1.map(fuse(bs, _)) ::: flats(rs2)
 | 
|  |    620 |     case r1 :: rs2 => r1 :: flats(rs2)
 | 
| 431 |    621 |   }
 | 
|  |    622 | 
 | 
| 492 |    623 | def distinctBy[B, C](xs: List[B], f: B => C, acc: List[C] = Nil): List[B] = xs match {
 | 
|  |    624 |   case Nil => Nil
 | 
|  |    625 |   case (x::xs) => {
 | 
|  |    626 |     val res = f(x)
 | 
|  |    627 |     if (acc.contains(res)) distinctBy(xs, f, acc)  
 | 
|  |    628 |     else x::distinctBy(xs, f, res::acc)
 | 
| 431 |    629 |   }
 | 
| 492 |    630 | } 
 | 
| 431 |    631 | 
 | 
|  |    632 | 
 | 
| 492 |    633 | def pruneRexp(r: ARexp, allowableTerms: List[Rexp]) : ARexp = {
 | 
|  |    634 |   r match {
 | 
|  |    635 |     case ASEQ(bs, r1, r2) => 
 | 
|  |    636 |       val termsTruncated = allowableTerms.collect(rt => rt match {
 | 
|  |    637 |         case SEQ(r1p, r2p) if(r2p == erase(r2)) => r1p//if(r2p == erase(r2)) 
 | 
|  |    638 |       })
 | 
|  |    639 |       val pruned : ARexp = pruneRexp(r1, termsTruncated)
 | 
|  |    640 |       pruned match {
 | 
|  |    641 |         case AZERO => AZERO
 | 
|  |    642 |         case AONE(bs1) => fuse(bs ++ bs1, r2)
 | 
|  |    643 |         case pruned1 => ASEQ(bs, pruned1, r2)
 | 
|  |    644 |       }
 | 
|  |    645 | 
 | 
|  |    646 |     case AALTS(bs, rs) => 
 | 
|  |    647 |       //allowableTerms.foreach(a => println(shortRexpOutput(a)))        
 | 
|  |    648 |       val rsp = rs.map(r => 
 | 
|  |    649 |                     pruneRexp(r, allowableTerms)
 | 
|  |    650 |                   )
 | 
|  |    651 |                   .filter(r => r != AZERO)
 | 
|  |    652 |       rsp match {
 | 
|  |    653 |         case Nil => AZERO
 | 
|  |    654 |         case r1::Nil => fuse(bs, r1)
 | 
|  |    655 |         case rs1 => AALTS(bs, rs1)
 | 
|  |    656 |       }
 | 
|  |    657 |     case r => 
 | 
|  |    658 |       if(allowableTerms.contains(erase(r))) r else AZERO //assert(r != AZERO)
 | 
|  |    659 |   }
 | 
|  |    660 | }
 | 
|  |    661 | 
 | 
|  |    662 | def oneSimp(r: Rexp) : Rexp = r match {
 | 
|  |    663 |   case SEQ(ONE, r) => r
 | 
|  |    664 |   case SEQ(r1, r2) => SEQ(oneSimp(r1), r2)
 | 
|  |    665 |   case r => r//assert r != 0 
 | 
| 432 |    666 |     
 | 
| 492 |    667 | }
 | 
| 431 |    668 | 
 | 
|  |    669 | 
 | 
| 492 |    670 | def distinctBy4(xs: List[ARexp], acc: List[Rexp] = Nil) : List[ARexp] = xs match {
 | 
|  |    671 |   case Nil => Nil
 | 
|  |    672 |   case x :: xs =>
 | 
|  |    673 |     //assert(acc.distinct == acc)
 | 
|  |    674 |     val erased = erase(x)
 | 
|  |    675 |     if(acc.contains(erased))
 | 
|  |    676 |       distinctBy4(xs, acc)
 | 
|  |    677 |     else{
 | 
|  |    678 |       val addToAcc =  breakIntoTerms(erased).filter(r => !acc.contains(oneSimp(r)))
 | 
|  |    679 |       //val xp = pruneRexp(x, addToAcc)
 | 
|  |    680 |       pruneRexp(x, addToAcc) match {
 | 
|  |    681 |         case AZERO => distinctBy4(xs, addToAcc.map(oneSimp(_)) ::: acc)
 | 
|  |    682 |         case xPrime => xPrime :: distinctBy4(xs, addToAcc.map(oneSimp(_)) ::: acc)
 | 
|  |    683 |       }
 | 
| 431 |    684 |     }
 | 
| 492 |    685 | }
 | 
|  |    686 | 
 | 
| 494 |    687 | // fun pAKC_aux :: "arexp list ⇒ arexp ⇒ rexp ⇒ arexp"
 | 
|  |    688 | //   where
 | 
|  |    689 | // "pAKC_aux rsa r ctx = (if (L (SEQ (erase r) ( ctx) )) ⊆ (L (erase (AALTs [] rsa))) then AZERO else
 | 
|  |    690 | //                           case r of (ASEQ bs r1 r2) ⇒ 
 | 
|  |    691 | //                             bsimp_ASEQ bs (pAKC_aux rsa r1 (SEQ  (erase r2) ( ctx) )) r2   |
 | 
|  |    692 | //                                     (AALTs bs rs) ⇒ 
 | 
|  |    693 | //                             bsimp_AALTs bs (flts (map (λr. pAKC_aux rsa r ( ctx) ) rs) )    |
 | 
|  |    694 | //                                     r             ⇒ r
 | 
|  |    695 | 
 | 
|  |    696 | // def canonicalSeq(rs: List[Rexp], acc: Rexp) = rs match {
 | 
|  |    697 | //   case r::Nil => SEQ(r, acc)
 | 
|  |    698 | //   case Nil => acc
 | 
|  |    699 | //   case r1::r2::Nil => SEQ(SEQ(r1, r2), acc)
 | 
|  |    700 | // }
 | 
|  |    701 | 
 | 
|  |    702 | 
 | 
|  |    703 | //the "fake" Language interpretation: just concatenates!
 | 
|  |    704 | def L(acc: Rexp, rs: List[Rexp]) : Rexp = rs match {
 | 
|  |    705 |   case Nil => acc
 | 
|  |    706 |   case r :: rs1 => 
 | 
| 500 |    707 |     // if(acc == ONE) 
 | 
|  |    708 |     //   L(r, rs1) 
 | 
|  |    709 |     // else
 | 
| 494 |    710 |       L(SEQ(acc, r), rs1)
 | 
|  |    711 | }
 | 
|  |    712 | 
 | 
| 500 |    713 | def rprint(r: Rexp) : Unit = println(shortRexpOutput(r))
 | 
| 526 |    714 | def rsprint(rs: Iterable[Rexp]) = rs.foreach(r => println(shortRexpOutput(r)))
 | 
|  |    715 | 
 | 
| 500 |    716 | def aprint(a: ARexp) = println(shortRexpOutput(erase(a)))
 | 
|  |    717 | def asprint(as: List[ARexp]) = as.foreach(a => println(shortRexpOutput(erase(a))))
 | 
|  |    718 | 
 | 
|  |    719 | def pAKC(acc: List[Rexp], r: ARexp, ctx: List[Rexp]) : ARexp = {
 | 
|  |    720 |   // println("pakc")
 | 
|  |    721 |   // println(shortRexpOutput(erase(r)))
 | 
|  |    722 |   // println("acc")
 | 
|  |    723 |   // rsprint(acc)
 | 
|  |    724 |   // println("ctx---------")
 | 
|  |    725 |   // rsprint(ctx)
 | 
|  |    726 |   // println("ctx---------end")
 | 
|  |    727 |   // rsprint(breakIntoTerms(L(erase(r), ctx)).map(oneSimp))
 | 
|  |    728 | 
 | 
|  |    729 |   if (breakIntoTerms(L(erase(r), ctx)).map(oneSimp).forall(acc.contains)) {//acc.flatMap(breakIntoTerms
 | 
| 494 |    730 |     AZERO
 | 
|  |    731 |   }
 | 
|  |    732 |   else{
 | 
|  |    733 |     r match {
 | 
|  |    734 |       case ASEQ(bs, r1, r2) => 
 | 
| 500 |    735 |       (pAKC(acc, r1, erase(r2) :: ctx)) match{
 | 
| 494 |    736 |         case AZERO => 
 | 
|  |    737 |           AZERO
 | 
|  |    738 |         case AONE(bs1) => 
 | 
|  |    739 |           fuse(bs1, r2)
 | 
|  |    740 |         case r1p => 
 | 
|  |    741 |           ASEQ(bs, r1p, r2)
 | 
|  |    742 |       }
 | 
|  |    743 |       case AALTS(bs, rs0) => 
 | 
|  |    744 |         // println("before pruning")
 | 
|  |    745 |         // println(s"ctx is ")
 | 
|  |    746 |         // ctx.foreach(r => println(shortRexpOutput(r)))
 | 
|  |    747 |         // println(s"rs0 is ")
 | 
|  |    748 |         // rs0.foreach(r => println(shortRexpOutput(erase(r))))
 | 
| 500 |    749 |         // println(s"acc is ")
 | 
|  |    750 |         // acc.foreach(r => println(shortRexpOutput(r)))
 | 
|  |    751 |         rs0.map(r => pAKC(acc, r, ctx)).filter(_ != AZERO) match {
 | 
| 494 |    752 |           case Nil => 
 | 
|  |    753 |             // println("after pruning Nil")
 | 
|  |    754 |             AZERO
 | 
|  |    755 |           case r :: Nil => 
 | 
|  |    756 |             // println("after pruning singleton")
 | 
|  |    757 |             // println(shortRexpOutput(erase(r)))
 | 
|  |    758 |             r 
 | 
|  |    759 |           case rs0p => 
 | 
|  |    760 |           // println("after pruning non-singleton")
 | 
|  |    761 |             AALTS(bs, rs0p)
 | 
|  |    762 |         }
 | 
|  |    763 |       case r => r
 | 
|  |    764 |     }
 | 
|  |    765 |   }
 | 
|  |    766 | }
 | 
|  |    767 | 
 | 
|  |    768 | def distinctBy5(xs: List[ARexp], acc: List[Rexp] = Nil) : List[ARexp] = xs match {
 | 
|  |    769 |   case Nil => 
 | 
|  |    770 |     Nil
 | 
|  |    771 |   case x :: xs => {
 | 
|  |    772 |     val erased = erase(x)
 | 
|  |    773 |     if(acc.contains(erased)){
 | 
|  |    774 |       distinctBy5(xs, acc)
 | 
|  |    775 |     }
 | 
|  |    776 |     else{
 | 
|  |    777 |       val pruned = pAKC(acc, x, Nil)
 | 
|  |    778 |       val newTerms = breakIntoTerms(erase(pruned))
 | 
|  |    779 |       pruned match {
 | 
|  |    780 |         case AZERO => 
 | 
|  |    781 |           distinctBy5(xs, acc)
 | 
|  |    782 |         case xPrime => 
 | 
|  |    783 |           xPrime :: distinctBy5(xs, newTerms.map(oneSimp) ::: acc)//distinctBy5(xs, addToAcc.map(oneSimp(_)) ::: acc)
 | 
|  |    784 |       }
 | 
|  |    785 |     }
 | 
|  |    786 |   }
 | 
|  |    787 | }
 | 
|  |    788 | 
 | 
| 532 |    789 | def atMostEmpty(r: Rexp) : Boolean = r match {
 | 
|  |    790 |   case ZERO => true
 | 
|  |    791 |   case ONE => true
 | 
|  |    792 |   case STAR(r) => atMostEmpty(r)
 | 
|  |    793 |   case SEQ(r1, r2) => atMostEmpty(r1) && atMostEmpty(r2)
 | 
|  |    794 |   case ALTS(r1, r2) => atMostEmpty(r1) && atMostEmpty(r2)
 | 
|  |    795 |   case CHAR(_) => false
 | 
|  |    796 | }
 | 
|  |    797 | 
 | 
|  |    798 | def isOne(r: Rexp) : Boolean = r match {
 | 
|  |    799 |   case ONE => true
 | 
|  |    800 |   case SEQ(r1, r2) => isOne(r1) && isOne(r2)
 | 
|  |    801 |   case ALTS(r1, r2) => (isOne(r1) || isOne(r2)) && (atMostEmpty(r1) && atMostEmpty(r2))//rs.forall(atMostEmpty) && rs.exists(isOne)
 | 
|  |    802 |   case STAR(r0) => atMostEmpty(r0)
 | 
|  |    803 |   case CHAR(c) => false
 | 
|  |    804 |   case ZERO => false
 | 
|  |    805 | 
 | 
|  |    806 | }
 | 
|  |    807 | 
 | 
| 526 |    808 | def strongBreakIntoTerms(r: Rexp): List[Rexp] = r match {
 | 
| 532 |    809 |   case SEQ(r1, r2)  => if(isOne(r1)) 
 | 
|  |    810 |                           //strongBreakIntoTerms(r1).map(r11 => SEQ(r11, r2)) ::: 
 | 
| 526 |    811 |                           strongBreakIntoTerms(r2) 
 | 
|  |    812 |                        else 
 | 
|  |    813 |                           strongBreakIntoTerms(r1).map(r11 => SEQ(r11, r2))
 | 
|  |    814 |   case ALTS(r1, r2) => strongBreakIntoTerms(r1) ::: strongBreakIntoTerms(r2)
 | 
|  |    815 |   case ZERO => Nil
 | 
|  |    816 |   case _ => r :: Nil
 | 
|  |    817 | }
 | 
|  |    818 | 
 | 
|  |    819 | def attachCtx(r: ARexp, ctx: List[Rexp]) : Set[Rexp] = {
 | 
|  |    820 |   val res = strongBreakIntoTerms((L(erase(r), ctx))).map(oneSimp)
 | 
|  |    821 |   res.toSet
 | 
| 518 |    822 | }
 | 
|  |    823 | 
 | 
| 530 |    824 | def ABIncludedByC[A, B, C](a: A, b: B, c: C, f: (A, B) => C, subseteqPred: (C, C) => Boolean) : Boolean = {
 | 
|  |    825 |   subseteqPred(f(a, b), c)
 | 
| 518 |    826 | }
 | 
| 532 |    827 | def rs1_subseteq_rs2(rs1: Set[Rexp], rs2: Set[Rexp]) : Boolean = {
 | 
| 526 |    828 |   val res = rs1.forall(rs2.contains)
 | 
|  |    829 |   res
 | 
| 518 |    830 | }
 | 
| 530 |    831 | def prune6(acc: Set[Rexp], r: ARexp, ctx: List[Rexp]) : ARexp = {
 | 
| 532 |    832 |   if (ABIncludedByC(r, ctx, acc, attachCtx, rs1_subseteq_rs2)) {//acc.flatMap(breakIntoTerms
 | 
| 518 |    833 |     AZERO
 | 
|  |    834 |   }
 | 
|  |    835 |   else{
 | 
|  |    836 |     r match {
 | 
|  |    837 |       case ASEQ(bs, r1, r2) => 
 | 
| 530 |    838 |       (prune6(acc, r1, erase(r2) :: ctx)) match{
 | 
| 518 |    839 |         case AZERO => 
 | 
|  |    840 |           AZERO
 | 
|  |    841 |         case AONE(bs1) => 
 | 
|  |    842 |           fuse(bs1, r2)
 | 
|  |    843 |         case r1p => 
 | 
|  |    844 |           ASEQ(bs, r1p, r2)
 | 
|  |    845 |       }
 | 
|  |    846 |       case AALTS(bs, rs0) => 
 | 
| 530 |    847 |         rs0.map(r => prune6(acc, r, ctx)).filter(_ != AZERO) match {
 | 
| 518 |    848 |           case Nil => 
 | 
|  |    849 |             AZERO
 | 
|  |    850 |           case r :: Nil => 
 | 
|  |    851 |             r 
 | 
|  |    852 |           case rs0p => 
 | 
|  |    853 |             AALTS(bs, rs0p)
 | 
|  |    854 |         }
 | 
|  |    855 |       case r => r
 | 
|  |    856 |     }
 | 
|  |    857 |   }
 | 
|  |    858 | }
 | 
|  |    859 | 
 | 
|  |    860 | 
 | 
| 526 |    861 | def distinctBy6(xs: List[ARexp], acc: Set[Rexp] = Set()) : List[ARexp] = xs match {
 | 
| 518 |    862 |   case Nil => 
 | 
|  |    863 |     Nil
 | 
|  |    864 |   case x :: xs => {
 | 
|  |    865 |     val erased = erase(x)
 | 
|  |    866 |     if(acc.contains(erased)){
 | 
|  |    867 |       distinctBy6(xs, acc)
 | 
|  |    868 |     }
 | 
|  |    869 |     else{
 | 
| 530 |    870 |       val pruned = prune6(acc, x, Nil)
 | 
| 526 |    871 |       val newTerms = strongBreakIntoTerms(erase(pruned))
 | 
| 518 |    872 |       pruned match {
 | 
|  |    873 |         case AZERO => 
 | 
|  |    874 |           distinctBy6(xs, acc)
 | 
|  |    875 |         case xPrime => 
 | 
| 526 |    876 |           xPrime :: distinctBy6(xs, newTerms.map(oneSimp) ++: acc)//distinctBy5(xs, addToAcc.map(oneSimp(_)) ::: acc)
 | 
| 518 |    877 |       }
 | 
|  |    878 |     }
 | 
|  |    879 |   }
 | 
|  |    880 | }
 | 
| 431 |    881 | 
 | 
| 492 |    882 | def breakIntoTerms(r: Rexp) : List[Rexp] = r match {
 | 
|  |    883 |   case SEQ(r1, r2)  => breakIntoTerms(r1).map(r11 => SEQ(r11, r2))
 | 
|  |    884 |   case ALTS(r1, r2) => breakIntoTerms(r1) ::: breakIntoTerms(r2)
 | 
| 494 |    885 |   case ZERO => Nil
 | 
| 492 |    886 |   case _ => r::Nil
 | 
|  |    887 | }
 | 
| 431 |    888 | 
 | 
|  |    889 | 
 | 
|  |    890 | 
 | 
| 492 |    891 | def decode_aux(r: Rexp, bs: Bits) : (Val, Bits) = (r, bs) match {
 | 
|  |    892 |   case (ONE, bs) => (Empty, bs)
 | 
|  |    893 |   case (CHAR(f), bs) => (Chr(f), bs)
 | 
|  |    894 |   case (ALTS(r1, r2), Z::bs1) => {
 | 
|  |    895 |       val (v, bs2) = decode_aux(r1, bs1)
 | 
|  |    896 |       (Left(v), bs2)
 | 
|  |    897 |   }
 | 
|  |    898 |   case (ALTS(r1, r2), S::bs1) => {
 | 
|  |    899 |       val (v, bs2) = decode_aux(r2, bs1)
 | 
|  |    900 |       (Right(v), bs2)
 | 
|  |    901 |   }
 | 
|  |    902 |   case (SEQ(r1, r2), bs) => {
 | 
|  |    903 |     val (v1, bs1) = decode_aux(r1, bs)
 | 
|  |    904 |     val (v2, bs2) = decode_aux(r2, bs1)
 | 
|  |    905 |     (Sequ(v1, v2), bs2)
 | 
|  |    906 |   }
 | 
|  |    907 |   case (STAR(r1), S::bs) => {
 | 
|  |    908 |     val (v, bs1) = decode_aux(r1, bs)
 | 
| 494 |    909 |     //(v)
 | 
| 492 |    910 |     val (Stars(vs), bs2) = decode_aux(STAR(r1), bs1)
 | 
|  |    911 |     (Stars(v::vs), bs2)
 | 
|  |    912 |   }
 | 
|  |    913 |   case (STAR(_), Z::bs) => (Stars(Nil), bs)
 | 
|  |    914 |   case (RECD(x, r1), bs) => {
 | 
|  |    915 |     val (v, bs1) = decode_aux(r1, bs)
 | 
|  |    916 |     (Rec(x, v), bs1)
 | 
|  |    917 |   }
 | 
|  |    918 |   case (NOT(r), bs) => (Nots(r.toString), bs)
 | 
| 431 |    919 | }
 | 
|  |    920 | 
 | 
| 492 |    921 | def decode(r: Rexp, bs: Bits) = decode_aux(r, bs) match {
 | 
|  |    922 |   case (v, Nil) => v
 | 
|  |    923 |   case _ => throw new Exception("Not decodable")
 | 
|  |    924 | }
 | 
|  |    925 | 
 | 
|  |    926 | 
 | 
|  |    927 | 
 | 
| 431 |    928 | def blexing_simp(r: Rexp, s: String) : Val = {
 | 
|  |    929 |     val bit_code = blex_simp(internalise(r), s.toList)
 | 
|  |    930 |     decode(r, bit_code)
 | 
| 492 |    931 | }
 | 
|  |    932 | def simpBlexer(r: Rexp, s: String) : Val = {
 | 
|  |    933 |   Try(blexing_simp(r, s)).getOrElse(Failure)
 | 
|  |    934 | }
 | 
| 431 |    935 | 
 | 
| 492 |    936 | def strong_blexing_simp(r: Rexp, s: String) : Val = {
 | 
|  |    937 |   decode(r, strong_blex_simp(internalise(r), s.toList))
 | 
|  |    938 | }
 | 
|  |    939 | 
 | 
| 494 |    940 | def strong_blexing_simp5(r: Rexp, s: String) : Val = {
 | 
|  |    941 |   decode(r, strong_blex_simp5(internalise(r), s.toList))
 | 
|  |    942 | }
 | 
|  |    943 | 
 | 
|  |    944 | 
 | 
| 492 |    945 | def strongBlexer(r: Rexp, s: String) : Val = {
 | 
|  |    946 |   Try(strong_blexing_simp(r, s)).getOrElse(Failure)
 | 
|  |    947 | }
 | 
| 431 |    948 | 
 | 
| 494 |    949 | def strongBlexer5(r: Rexp, s: String): Val = {
 | 
|  |    950 |   Try(strong_blexing_simp5(r, s)).getOrElse(Failure)
 | 
|  |    951 | }
 | 
|  |    952 | 
 | 
| 492 |    953 | def strong_blex_simp(r: ARexp, s: List[Char]) : Bits = s match {
 | 
|  |    954 |   case Nil => {
 | 
|  |    955 |     if (bnullable(r)) {
 | 
|  |    956 |       //println(asize(r))
 | 
|  |    957 |       val bits = mkepsBC(r)
 | 
|  |    958 |       bits
 | 
| 431 |    959 |     }
 | 
| 492 |    960 |     else 
 | 
|  |    961 |       throw new Exception("Not matched")
 | 
| 431 |    962 |   }
 | 
| 492 |    963 |   case c::cs => {
 | 
|  |    964 |     val der_res = bder(c,r)
 | 
|  |    965 |     val simp_res = strongBsimp(der_res)  
 | 
|  |    966 |     strong_blex_simp(simp_res, cs)      
 | 
|  |    967 |   }
 | 
|  |    968 | }
 | 
| 431 |    969 | 
 | 
| 494 |    970 | def strong_blex_simp5(r: ARexp, s: List[Char]) : Bits = s match {
 | 
|  |    971 |   case Nil => {
 | 
|  |    972 |     if (bnullable(r)) {
 | 
|  |    973 |       val bits = mkepsBC(r)
 | 
|  |    974 |       bits
 | 
|  |    975 |     }
 | 
|  |    976 |     else 
 | 
|  |    977 |       throw new Exception("Not matched")
 | 
|  |    978 |   }
 | 
|  |    979 |   case c::cs => {
 | 
|  |    980 |     val der_res = bder(c,r)
 | 
|  |    981 |     val simp_res = strongBsimp5(der_res)  
 | 
|  |    982 |     strong_blex_simp5(simp_res, cs)      
 | 
|  |    983 |   }
 | 
|  |    984 | }
 | 
| 431 |    985 | 
 | 
|  |    986 | 
 | 
|  |    987 |   def bders_simp(s: List[Char], r: ARexp) : ARexp = s match {
 | 
|  |    988 |     case Nil => r
 | 
| 435 |    989 |     case c::s => 
 | 
| 494 |    990 |       //println(erase(r))
 | 
| 435 |    991 |       bders_simp(s, bsimp(bder(c, r)))
 | 
| 431 |    992 |   }
 | 
|  |    993 |   
 | 
| 494 |    994 |   def bdersStrong5(s: List[Char], r: ARexp) : ARexp = s match {
 | 
|  |    995 |     case Nil => r
 | 
|  |    996 |     case c::s => bdersStrong5(s, strongBsimp5(bder(c, r)))
 | 
|  |    997 |   }
 | 
| 518 |    998 |   def bdersStrong6(s: List[Char], r: ARexp) : ARexp = s match {
 | 
|  |    999 |     case Nil => r
 | 
|  |   1000 |     case c::s => bdersStrong6(s, strongBsimp6(bder(c, r)))
 | 
|  |   1001 |   }
 | 
| 532 |   1002 |   def bdersStrong7(s: List[Char], r: ARexp) : ARexp = s match {
 | 
|  |   1003 |     case Nil => r
 | 
|  |   1004 |     case c::s => bdersStrong7(s, strongBsimp7(bder(c, r)))
 | 
|  |   1005 |   }
 | 
| 431 |   1006 |   def bdersSimp(s: String, r: Rexp) : ARexp = bders_simp(s.toList, internalise(r))
 | 
|  |   1007 | 
 | 
| 492 |   1008 |   def bdersStrong(s: List[Char], r: ARexp) : ARexp = s match {
 | 
| 431 |   1009 |     case Nil => r 
 | 
| 492 |   1010 |     case c::s => bdersStrong(s, strongBsimp(bder(c, r)))
 | 
| 431 |   1011 |   }
 | 
|  |   1012 | 
 | 
| 492 |   1013 |   def bdersStrongRexp(s: String, r: Rexp) : ARexp = bdersStrong(s.toList, internalise(r))
 | 
| 431 |   1014 | 
 | 
|  |   1015 |   def erase(r:ARexp): Rexp = r match{
 | 
|  |   1016 |     case AZERO => ZERO
 | 
|  |   1017 |     case AONE(_) => ONE
 | 
|  |   1018 |     case ACHAR(bs, c) => CHAR(c)
 | 
|  |   1019 |     case AALTS(bs, Nil) => ZERO
 | 
|  |   1020 |     case AALTS(bs, a::Nil) => erase(a)
 | 
|  |   1021 |     case AALTS(bs, a::as) => ALTS(erase(a), erase(AALTS(bs, as)))
 | 
|  |   1022 |     case ASEQ(bs, r1, r2) => SEQ (erase(r1), erase(r2))
 | 
|  |   1023 |     case ASTAR(cs, r)=> STAR(erase(r))
 | 
|  |   1024 |     case ANOT(bs, r) => NOT(erase(r))
 | 
|  |   1025 |     case AANYCHAR(bs) => ANYCHAR
 | 
|  |   1026 |   }
 | 
|  |   1027 | 
 | 
|  |   1028 | 
 | 
| 492 |   1029 |   def allCharSeq(r: Rexp) : Boolean = r match {
 | 
|  |   1030 |     case CHAR(c) => true
 | 
|  |   1031 |     case SEQ(r1, r2) => allCharSeq(r1) && allCharSeq(r2)
 | 
|  |   1032 |     case _ => false
 | 
|  |   1033 |   }
 | 
|  |   1034 | 
 | 
|  |   1035 |   def flattenSeq(r: Rexp) : String = r match {
 | 
|  |   1036 |     case CHAR(c) => c.toString
 | 
|  |   1037 |     case SEQ(r1, r2) => flattenSeq(r1) ++ flattenSeq(r2)
 | 
|  |   1038 |     case _ => throw new Error("flatten unflattenable rexp")
 | 
|  |   1039 |   } 
 | 
| 431 |   1040 | 
 | 
| 492 |   1041 |   def shortRexpOutput(r: Rexp) : String = r match {
 | 
|  |   1042 |       case CHAR(c) => c.toString
 | 
|  |   1043 |       case ONE => "1"
 | 
|  |   1044 |       case ZERO => "0"
 | 
|  |   1045 |       case SEQ(r1, r2) if(allCharSeq(r)) => flattenSeq(r)//"[" ++ shortRexpOutput(r1) ++ "~" ++ shortRexpOutput(r2) ++ "]"
 | 
|  |   1046 |       case SEQ(r1, r2) => "[" ++ shortRexpOutput(r1) ++ "~" ++ shortRexpOutput(r2) ++ "]"
 | 
|  |   1047 |       case ALTS(r1, r2) => "(" ++ shortRexpOutput(r1) ++ "+" ++ shortRexpOutput(r2) ++ ")"
 | 
|  |   1048 |       case STAR(STAR(r)) => "(..)*"// ++ shortRexpOutput(r) ++ "]*"
 | 
|  |   1049 |       case STAR(r) => "STAR(" ++ shortRexpOutput(r) ++ ")"
 | 
|  |   1050 |       //case RTOP => "RTOP"
 | 
|  |   1051 |     }
 | 
|  |   1052 | 
 | 
| 431 |   1053 | 
 | 
| 492 |   1054 |   def blex_simp(r: ARexp, s: List[Char]) : Bits = s match {
 | 
|  |   1055 |       case Nil => {
 | 
|  |   1056 |         if (bnullable(r)) {
 | 
|  |   1057 |           val bits = mkepsBC(r)
 | 
|  |   1058 |           bits
 | 
|  |   1059 |         }
 | 
|  |   1060 |         else 
 | 
|  |   1061 |           throw new Exception("Not matched")
 | 
|  |   1062 |       }
 | 
|  |   1063 |       case c::cs => {
 | 
|  |   1064 |         val der_res = bder(c,r)
 | 
|  |   1065 |         val simp_res = bsimp(der_res)  
 | 
|  |   1066 |         blex_simp(simp_res, cs)      
 | 
|  |   1067 |       }
 | 
| 431 |   1068 |   }
 | 
|  |   1069 | 
 | 
|  |   1070 | 
 | 
| 492 |   1071 | 
 | 
|  |   1072 | 
 | 
|  |   1073 |     def size(r: Rexp) : Int = r match {
 | 
|  |   1074 |       case ZERO => 1
 | 
|  |   1075 |       case ONE => 1
 | 
|  |   1076 |       case CHAR(_) => 1
 | 
|  |   1077 |       case ANYCHAR => 1
 | 
|  |   1078 |       case NOT(r0) => 1 + size(r0)
 | 
|  |   1079 |       case SEQ(r1, r2) => 1 + size(r1) + size(r2)
 | 
|  |   1080 |       case ALTS(r1, r2) => 1 + List(r1, r2).map(size).sum
 | 
|  |   1081 |       case STAR(r) => 1 + size(r)
 | 
| 431 |   1082 |     }
 | 
|  |   1083 | 
 | 
| 492 |   1084 |     def asize(a: ARexp) = size(erase(a))
 | 
| 431 |   1085 | 
 | 
|  |   1086 | //pder related
 | 
|  |   1087 | type Mon = (Char, Rexp)
 | 
|  |   1088 | type Lin = Set[Mon]
 | 
|  |   1089 | 
 | 
|  |   1090 | def dot_prod(rs: Set[Rexp], r: Rexp): Set[Rexp] = r match {
 | 
|  |   1091 |     case ZERO => Set()
 | 
|  |   1092 |     case ONE => rs
 | 
|  |   1093 |     case r => rs.map((re) => if (re == ONE) r else SEQ(re, r)  )   
 | 
|  |   1094 |   }
 | 
|  |   1095 |   def cir_prod(l: Lin, t: Rexp): Lin = t match {//remember this Lin is different from the Lin in Antimirov's paper. Here it does not mean the set of all subsets of linear forms that does not contain zero, but rather the type a set of linear forms
 | 
|  |   1096 |     case ZERO => Set()
 | 
|  |   1097 |     case ONE => l
 | 
| 526 |   1098 |     case t => l.map( m => m._2 match 
 | 
|  |   1099 |       {
 | 
|  |   1100 |         case ZERO => m 
 | 
|  |   1101 |         case ONE => (m._1, t) 
 | 
|  |   1102 |         case p => (m._1, SEQ(p, t)) 
 | 
|  |   1103 |       }  
 | 
|  |   1104 |     
 | 
|  |   1105 |     )
 | 
| 431 |   1106 |   }
 | 
|  |   1107 |   def lf(r: Rexp): Lin = r match {
 | 
|  |   1108 |     case ZERO => Set()
 | 
|  |   1109 |     case ONE => Set()
 | 
|  |   1110 |     case CHAR(f) => {
 | 
|  |   1111 |       //val Some(c) = alphabet.find(f) 
 | 
|  |   1112 |       Set((f, ONE))
 | 
|  |   1113 |     }
 | 
|  |   1114 |     case ALTS(r1, r2) => {
 | 
|  |   1115 |       lf(r1 ) ++ lf(r2)
 | 
|  |   1116 |     }
 | 
|  |   1117 |     case STAR(r1) => cir_prod(lf(r1), STAR(r1)) //may try infix notation later......
 | 
|  |   1118 |     case SEQ(r1, r2) =>{
 | 
|  |   1119 |       if (nullable(r1))
 | 
|  |   1120 |         cir_prod(lf(r1), r2) ++ lf(r2)
 | 
|  |   1121 |       else
 | 
|  |   1122 |         cir_prod(lf(r1), r2) 
 | 
|  |   1123 |     }
 | 
|  |   1124 |   }
 | 
|  |   1125 |   def lfs(r: Set[Rexp]): Lin = {
 | 
|  |   1126 |     r.foldLeft(Set[Mon]())((acc, r) => acc ++ lf(r))
 | 
|  |   1127 |   }
 | 
|  |   1128 | 
 | 
|  |   1129 |   def pder(x: Char, t: Rexp): Set[Rexp] = {
 | 
|  |   1130 |     val lft = lf(t)
 | 
|  |   1131 |     (lft.filter(mon => if(mon._1 == x) true else false)).map(mon => mon._2)
 | 
|  |   1132 |   }
 | 
|  |   1133 |   def pders_single(s: List[Char], t: Rexp) : Set[Rexp] = s match {
 | 
|  |   1134 |     case x::xs => pders(xs, pder(x, t))
 | 
|  |   1135 |     case Nil => Set(t)
 | 
|  |   1136 |   }
 | 
|  |   1137 |   def pders(s: List[Char], ts: Set[Rexp]) : Set[Rexp] = s match {
 | 
|  |   1138 |     case x::xs => pders(xs, ts.foldLeft(Set[Rexp]())((acc, t) => acc ++ pder(x, t)))
 | 
|  |   1139 |     case Nil => ts 
 | 
|  |   1140 |   }
 | 
| 526 |   1141 |   def pderss(ss: List[List[Char]], t: Rexp): Set[Rexp] = 
 | 
|  |   1142 |     ss.foldLeft( Set[Rexp]() )( (acc, s) => pders_single(s, t) ++ acc )
 | 
| 431 |   1143 |   def pdera(t: Rexp): Set[Rexp] = lf(t).map(mon => mon._2)
 | 
|  |   1144 |   //all implementation of partial derivatives that involve set union are potentially buggy
 | 
|  |   1145 |   //because they don't include the original regular term before they are pdered.
 | 
|  |   1146 |   //now only pderas is fixed.
 | 
| 526 |   1147 |   def pderas(t: Set[Rexp], d: Int): Set[Rexp] = 
 | 
|  |   1148 |     if(d > 0) 
 | 
|  |   1149 |       pderas(lfs(t).map(mon => mon._2), d - 1) ++ t 
 | 
|  |   1150 |     else 
 | 
|  |   1151 |       lfs(t).map(mon => mon._2) ++ t//repeated application of pderas over the newest set of pders.
 | 
| 431 |   1152 |   def pderUNIV(r: Rexp) : Set[Rexp] = pderas(Set(r), awidth(r) + 1)
 | 
|  |   1153 |   def awidth(r: Rexp) : Int = r match {
 | 
|  |   1154 |     case CHAR(c) => 1
 | 
|  |   1155 |     case SEQ(r1, r2) => awidth(r1) + awidth(r2)
 | 
|  |   1156 |     case ALTS(r1, r2) => awidth(r1) + awidth(r2)
 | 
|  |   1157 |     case ONE => 0
 | 
|  |   1158 |     case ZERO => 0
 | 
|  |   1159 |     case STAR(r) => awidth(r)
 | 
|  |   1160 |   }
 | 
|  |   1161 |   //def sigma_lf(l: Set[Mon]) : Rexp = ALTS(l.map(mon => SEQ(CHAR(mon._1),mon._2)).toList)
 | 
|  |   1162 |   //def sigma(rs: Set[Rexp]) : Rexp = ALTS(rs.toList)
 | 
|  |   1163 |   def o(r: Rexp) = if (nullable(r)) ONE else ZERO
 | 
|  |   1164 |   //def nlf(t: Rexp) : Rexp = ALTS(List( o(t), sigma_lf(lf(t)) ))
 | 
|  |   1165 |   def pdp(x: Char, r: Rexp) : Set[Rexp] = r match {
 | 
|  |   1166 |     case ZERO => Set[Rexp]()
 | 
|  |   1167 |     case ONE => Set[Rexp]()
 | 
|  |   1168 |     case CHAR(f) => if(x == f) Set(ONE) else Set[Rexp]()
 | 
|  |   1169 |     case ALTS(r1, r2) => pdp(x, r1) ++ pdp(x, r2)
 | 
|  |   1170 |     case STAR(r1) => pdp(x, r).map(a => SEQ(a, STAR(r1)))
 | 
|  |   1171 |     case SEQ(a0, b) => if(nullable(a0)) pdp(x, a0).map(a => SEQ(a, b)) ++ pdp(x, b) else pdp(x, a0).map(a => SEQ(a, b))
 | 
|  |   1172 |   }
 | 
|  |   1173 |   def pdps(s: List[Char], ts: Set[Rexp]): Set[Rexp] = s match {
 | 
|  |   1174 |     case x::xs => pdps(xs, ts.foldLeft(Set[Rexp]())((acc, t) => acc ++ pder(x, t)))
 | 
|  |   1175 |     case Nil => ts   
 | 
|  |   1176 |   }
 | 
|  |   1177 |   def pdpss(ss: List[List[Char]], t: Rexp): Set[Rexp] = ss.foldLeft( Set[Rexp]())((acc, s) => pdps(s, Set(t)) ++ acc)
 | 
|  |   1178 | 
 | 
|  |   1179 | 
 | 
|  |   1180 | 
 | 
|  |   1181 | def starPrint(r: Rexp) : Unit = r match {
 | 
|  |   1182 |         
 | 
|  |   1183 |           case SEQ(head, rstar) =>
 | 
|  |   1184 |             println(shortRexpOutput(head) ++ "~STARREG")
 | 
|  |   1185 |           case STAR(rstar) =>
 | 
|  |   1186 |             println("STARREG")
 | 
|  |   1187 |           case ALTS(r1, r2) =>  
 | 
|  |   1188 |             println("(")
 | 
|  |   1189 |             starPrint(r1)
 | 
|  |   1190 |             println("+")
 | 
|  |   1191 |             starPrint(r2)
 | 
|  |   1192 |             println(")")
 | 
|  |   1193 |           case ZERO => println("0")
 | 
|  |   1194 |       }
 | 
|  |   1195 | 
 | 
|  |   1196 | // @arg(doc = "small tests")
 | 
| 516 |   1197 | def n_astar_list(d: Int) : Rexp = {
 | 
|  |   1198 |   if(d == 0) STAR("a") 
 | 
|  |   1199 |   else ALTS(STAR("a" * d), n_astar_list(d - 1))
 | 
|  |   1200 | }
 | 
|  |   1201 | def n_astar_alts(d: Int) : Rexp = d match {
 | 
|  |   1202 |   case 0 => n_astar_list(0)
 | 
|  |   1203 |   case d => STAR(n_astar_list(d))
 | 
|  |   1204 |   // case r1 :: r2 :: Nil => ALTS(r1, r2)
 | 
|  |   1205 |   // case r1 :: Nil => r1
 | 
|  |   1206 |   // case r :: rs => ALTS(r, n_astar_alts(rs))
 | 
|  |   1207 |   // case Nil => throw new Error("should give at least 1 elem")
 | 
|  |   1208 | }
 | 
|  |   1209 | def n_astar_aux(d: Int) = {
 | 
|  |   1210 |   if(d == 0) n_astar_alts(0)
 | 
|  |   1211 |   else ALTS(n_astar_alts(d), n_astar_alts(d - 1))
 | 
|  |   1212 | }
 | 
|  |   1213 | 
 | 
|  |   1214 | def n_astar(d: Int) : Rexp = STAR(n_astar_aux(d))
 | 
|  |   1215 | //val STARREG = n_astar(3)
 | 
|  |   1216 | // ( STAR("a") | 
 | 
|  |   1217 | //                  ("a" | "aa").% | 
 | 
|  |   1218 | //                 ( "a" | "aa" | "aaa").% 
 | 
|  |   1219 | //                 ).%
 | 
|  |   1220 |                 //( "a" | "aa" | "aaa" | "aaaa").% |
 | 
|  |   1221 |                 //( "a" | "aa" | "aaa" | "aaaa" | "aaaaa").% 
 | 
| 431 |   1222 | (((STAR("a") | ( STAR("aaa")) | STAR("aaaaa"| ( STAR("aaaaaaa")) | STAR("aaaaaaaaaaa"))).%).%).%
 | 
|  |   1223 | 
 | 
|  |   1224 | // @main
 | 
| 492 |   1225 | 
 | 
| 516 |   1226 | def lcm(list: Seq[Int]):Int=list.foldLeft(1:Int){
 | 
|  |   1227 |   (a, b) => b * a /
 | 
|  |   1228 |   Stream.iterate((a,b)){case (x,y) => (y, x%y)}.dropWhile(_._2 != 0).head._1.abs
 | 
|  |   1229 | }
 | 
| 492 |   1230 | 
 | 
| 431 |   1231 | def small() = {
 | 
| 516 |   1232 |   //val pderSTAR = pderUNIV(STARREG)
 | 
| 492 |   1233 | 
 | 
| 516 |   1234 |   //val refSize = pderSTAR.map(size(_)).sum
 | 
| 518 |   1235 |   for(n <- 5 to 5){
 | 
| 516 |   1236 |     val STARREG = n_astar(n)
 | 
|  |   1237 |     val iMax = (lcm((1 to n).toList))
 | 
| 518 |   1238 |     for(i <- 1 to iMax + 2){// 100, 400, 800, 840, 841, 900 
 | 
| 516 |   1239 |       val prog0 = "a" * i
 | 
|  |   1240 |       //println(s"test: $prog0")
 | 
| 518 |   1241 |       print(i)
 | 
| 516 |   1242 |       print(" ")
 | 
|  |   1243 |       // print(i)
 | 
|  |   1244 |       // print(" ")
 | 
|  |   1245 |       println(asize(bders_simp(prog0.toList, internalise(STARREG))))
 | 
|  |   1246 |     }
 | 
| 492 |   1247 |   }
 | 
| 431 |   1248 | }
 | 
|  |   1249 | 
 | 
| 492 |   1250 | def generator_test() {
 | 
|  |   1251 | 
 | 
| 532 |   1252 |   test(rexp(4), 1000000) { (r: Rexp) => 
 | 
| 500 |   1253 |   // ALTS(SEQ(SEQ(ONE,CHAR('a')),STAR(CHAR('a'))),SEQ(ALTS(CHAR('c'),ONE),STAR(ZERO))))))), 1) { (r: Rexp) => 
 | 
| 532 |   1254 |     val ss = Set("b")//stringsFromRexp(r)
 | 
| 518 |   1255 |     val boolList = ss.filter(s => s != "").map(s => {
 | 
|  |   1256 |       //val bdStrong = bdersStrong(s.toList, internalise(r))
 | 
| 532 |   1257 |       val bdStrong6 = bdersStrong7(s.toList, internalise(r))
 | 
|  |   1258 |       val bdStrong6Set = strongBreakIntoTerms(erase(bdStrong6))
 | 
|  |   1259 |       val pdersSet = pderUNIV(r)//.flatMap(r => strongBreakIntoTerms(r))
 | 
|  |   1260 |       val pdersSetBroken = pdersSet.flatMap(r => strongBreakIntoTerms(r))
 | 
|  |   1261 |       bdStrong6Set.size <= pdersSet.size || bdStrong6Set.size <= pdersSetBroken.size
 | 
| 493 |   1262 |     })
 | 
| 532 |   1263 |     //println(boolList)
 | 
| 500 |   1264 |     //!boolList.exists(b => b == false)
 | 
| 493 |   1265 |     !boolList.exists(b => b == false)
 | 
| 492 |   1266 |   }
 | 
|  |   1267 | }
 | 
| 518 |   1268 | // small()
 | 
| 532 |   1269 | //  generator_test()
 | 
|  |   1270 |   
 | 
|  |   1271 |   
 | 
|  |   1272 |   //STAR(STAR(STAR(SEQ(SEQ(ALTS(STAR(ALTS(ONE,CHAR('c'))),
 | 
|  |   1273 |           //  CHAR('c')),ALTS(CHAR('a'),ALTS(STAR(CHAR('b')),ALTS(CHAR('a'),ZERO)))),
 | 
|  |   1274 |           //  CHAR('c')))))//SEQ(STAR(CHAR('c')),STAR(SEQ(STAR(CHAR('c')),ONE)))//STAR(SEQ(ALTS(STAR(CHAR('c')),CHAR('c')),SEQ(ALTS(CHAR('c'),ONE),ONE)))
 | 
|  |   1275 | //counterexample1: STAR(SEQ(ALTS(STAR(ZERO),ALTS(CHAR(a),CHAR(b))),SEQ(ONE,ALTS(CHAR(a),CHAR(b)))))
 | 
|  |   1276 | //counterexample2: SEQ(ALTS(SEQ(CHAR(a),STAR(ONE)),STAR(ONE)),ALTS(CHAR(a),SEQ(ALTS(CHAR(c),CHAR(a)),CHAR(b))))
 | 
| 518 |   1277 | def counterexample_check() {
 | 
| 532 |   1278 |   val r = SEQ(SEQ(STAR(ALTS(CHAR('a'),CHAR('b'))),
 | 
|  |   1279 |     ALTS(ALTS(CHAR('c'),CHAR('b')),STAR(ONE))),STAR(CHAR('b')))
 | 
|  |   1280 |   val s = "b"
 | 
|  |   1281 |   val bdStrong5 = bdersStrong7(s.toList, internalise(r))
 | 
| 518 |   1282 |   val bdStrong5Set = breakIntoTerms(erase(bdStrong5))
 | 
| 532 |   1283 |   val pdersSet = pderUNIV(r)//.map(r => erase(bsimp(internalise(r))))//.flatMap(r => strongBreakIntoTerms(r))//.map(oneSimp).flatMap(r => breakIntoTerms(r))
 | 
| 518 |   1284 |   println("original regex ")
 | 
|  |   1285 |   rprint(r)
 | 
|  |   1286 |   println("after strong bsimp")
 | 
|  |   1287 |   aprint(bdStrong5)
 | 
|  |   1288 |   println("turned into a set %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%   ")
 | 
|  |   1289 |   rsprint(bdStrong5Set)
 | 
|  |   1290 |   println("after pderUNIV")
 | 
|  |   1291 |   rsprint(pdersSet.toList)
 | 
| 532 |   1292 | 
 | 
| 518 |   1293 | }
 | 
| 532 |   1294 | counterexample_check()
 | 
|  |   1295 | 
 | 
| 526 |   1296 | def linform_test() {
 | 
| 530 |   1297 |   val r = STAR(SEQ(STAR(CHAR('c')),ONE))//SEQ(STAR(CHAR('c')),STAR(SEQ(STAR(CHAR('c')),ONE))) //
 | 
| 526 |   1298 |   val r_linforms = lf(r)
 | 
|  |   1299 |   println(r_linforms.size)
 | 
| 530 |   1300 |   val pderuniv = pderUNIV(r)
 | 
|  |   1301 |   println(pderuniv.size)
 | 
| 526 |   1302 | }
 | 
| 530 |   1303 | // linform_test()
 | 
| 516 |   1304 | // 1
 | 
| 518 |   1305 | def newStrong_test() {
 | 
|  |   1306 |   val r2 = (CHAR('b') | ONE)
 | 
|  |   1307 |   val r0 = CHAR('d')
 | 
|  |   1308 |   val r1 = (ONE | CHAR('c'))
 | 
|  |   1309 |   val expRexp = (SEQ(r2, r0) | SEQ(SEQ(r1, r2), r0))
 | 
|  |   1310 |   println(s"original regex is: ")
 | 
|  |   1311 |   rprint(expRexp)
 | 
|  |   1312 |   val expSimp5 = strongBsimp5(internalise(expRexp))
 | 
|  |   1313 |   val expSimp6 = strongBsimp6(internalise(expRexp))
 | 
|  |   1314 |   aprint(expSimp5)
 | 
|  |   1315 |   aprint(expSimp6)
 | 
|  |   1316 | }
 | 
|  |   1317 | // newStrong_test()
 | 
| 516 |   1318 | // SEQ(SEQ(SEQ(ONE,CHAR('b')),STAR(CHAR('b'))),
 | 
|  |   1319 | // SEQ(ALTS(ALTS(ZERO,STAR(CHAR('b'))),
 | 
|  |   1320 | // STAR(ALTS(CHAR('a'),SEQ(SEQ(STAR(ALTS(STAR(CHAR('c')),CHAR('a'))),
 | 
|  |   1321 | // SEQ(CHAR('a'),SEQ(ALTS(CHAR('b'),ZERO),SEQ(ONE,CHAR('b'))))),ONE)))),ONE))
 | 
| 493 |   1322 | 
 | 
|  |   1323 | 
 | 
|  |   1324 | // Sequ(Sequ(Sequ(Empty,Chr(b)),Stars(List(Chr(b), Chr(b)))),Sequ(Right(Stars(List(Right(Sequ(Sequ(Stars(List(Right(Chr(a)), Right(Chr(a)))),Sequ(Chr(a),Sequ(Left(Chr(b)),Sequ(Empty,Chr(b))))),Empty)), Right(Sequ(Sequ(Stars(List(Right(Chr(a)), Right(Chr(a)))),Sequ(Chr(a),Sequ(Left(Chr(b)),Sequ(Empty,Chr(b))))),Empty))))),Empty))
 | 
|  |   1325 | // Sequ(Sequ(Sequ(Empty,Chr(b)),Stars(List(Chr(b), Chr(b)))),Sequ(Right(Stars(List(Right(Sequ(Sequ(Stars(List(Right(Chr(a)), Right(Chr(a)))),Sequ(Chr(a),Sequ(Left(Chr(b)),Sequ(Empty,Chr(b))))),Empty)), Right(Sequ(Sequ(Stars(List(Right(Chr(a)), Right(Chr(a)))),Sequ(Chr(a),Sequ(Left(Chr(b)),Sequ(Empty,Chr(b))))),Empty))))),Empty)) |