Matcher.thy
changeset 102 5fed809d0fc1
parent 24 f72c82bf59e5
child 103 f460d5f75cb5
--- a/Matcher.thy	Mon Feb 14 09:38:18 2011 +0000
+++ b/Matcher.thy	Mon Feb 14 11:12:01 2011 +0000
@@ -38,6 +38,14 @@
 | STAR rexp
 
 
+definition
+  "DERIV s A \<equiv> {s'. s @ s' \<in> A}"
+
+definition
+  "delta A = (if [] \<in> A then {[]} else {})"
+
+
+
 section {* Semantics of Regular Expressions *}
  
 fun