// Version which attempts to move whole strings, not// just characters, under derivatives whenever possibleabstract class Rexpcase object ZERO extends Rexpcase object ONE extends Rexpcase class CHAR(c: Char) extends Rexpcase class ALT(r1: Rexp, r2: Rexp) extends Rexp case class SEQ(r1: Rexp, r2: Rexp) extends Rexp case class STAR(r: Rexp) extends Rexp case class NTIMES(r: Rexp, n: Int) extends Rexp // nullable function: tests whether the regular // expression can recognise the empty stringdef nullable (r: Rexp) : Boolean = r match { case ZERO => false case ONE => true case CHAR(_) => false case ALT(r1, r2) => nullable(r1) || nullable(r2) case SEQ(r1, r2) => nullable(r1) && nullable(r2) case STAR(_) => true case NTIMES(r, i) => if (i == 0) true else nullable(r)}// derivative of a regular expression w.r.t. a characterdef der (c: Char, r: Rexp) : Rexp = r match { case ZERO => ZERO case ONE => ZERO case CHAR(d) => if (c == d) ONE else ZERO case ALT(r1, r2) => ALT(der(c, r1), der(c, r2)) case SEQ(r1, r2) => if (nullable(r1)) ALT(SEQ(der(c, r1), r2), der(c, r2)) else SEQ(der(c, r1), r2) case STAR(r1) => SEQ(der(c, r1), STAR(r1)) case NTIMES(r1, i) => if (i == 0) ZERO else der(c, SEQ(r1, NTIMES(r1, i - 1)))}def simp(r: Rexp) : Rexp = r match { case ALT(r1, r2) => (simp(r1), simp(r2)) match { case (ZERO, r2s) => r2s case (r1s, ZERO) => r1s case (r1s, r2s) => if (r1s == r2s) r1s else ALT (r1s, r2s) } case SEQ(r1, r2) => (simp(r1), simp(r2)) match { case (ZERO, _) => ZERO case (_, ZERO) => ZERO case (ONE, r2s) => r2s case (r1s, ONE) => r1s case (r1s, r2s) => SEQ(r1s, r2s) } case r => r}//exampleval r = SEQ(SEQ(CHAR('x'), CHAR('y')), CHAR('z'))der('x', r)der('y', der('x', r))der('z', der('y', der('x', r)))simp(der('z', der('y', der('x', r))))// *new*// derivative w.r.t. a string (iterates der)def ders2(s: List[Char], r: Rexp) : Rexp = (s, r) match { case (Nil, r) => r case (s, ZERO) => ZERO case (s, ONE) => if (s == Nil) ONE else ZERO case (s, CHAR(c)) => if (s == List(c)) ONE else if (s == Nil) CHAR(c) else ZERO case (s, ALT(r1, r2)) => ALT(ders2(s, r1), ders2(s, r2)) case (c::s, r) => ders2(s, simp(der(c, r)))}// main matcher functiondef matcher(r: Rexp, s: String) : Boolean = nullable(ders2(s.toList, r))//one or zerodef OPT(r: Rexp) = ALT(r, ONE)// Test Casesdef EVIL1(n: Int) = SEQ(NTIMES(OPT(CHAR('a')), n), NTIMES(CHAR('a'), n))val EVIL2 = SEQ(STAR(STAR(CHAR('a'))), CHAR('b'))def time_needed[T](i: Int, code: => T) = { val start = System.nanoTime() for (j <- 1 to i) code val end = System.nanoTime() (end - start)/(i * 1.0e9)}//test: (a?{n}) (a{n})for (i <- 1 to 7000001 by 500000) { println(i + " " + "%.5f".format(time_needed(2, matcher(EVIL1(i), "a" * i))))}for (i <- 1 to 7000001 by 500000) { println(i + " " + "%.5f".format(time_needed(2, matcher(EVIL1(i), "a" * i))))}//test: (a*)* bfor (i <- 1 to 7000001 by 500000) { println(i + " " + "%.5f".format(time_needed(2, matcher(EVIL2, "a" * i))))}for (i <- 1 to 7000001 by 500000) { println(i + " " + "%.5f".format(time_needed(2, matcher(EVIL2, "a" * i))))}