src/HOL/Lex/RegExp2NA.thy
changeset 8732 aef229ca5e77
parent 7224 e41e64476f9b
child 10834 a7897aebbffc
--- a/src/HOL/Lex/RegExp2NA.thy	Mon Apr 17 14:27:10 2000 +0200
+++ b/src/HOL/Lex/RegExp2NA.thy	Tue Apr 18 00:36:02 2000 +0200
@@ -7,7 +7,7 @@
 into nondeterministic automata *without* epsilon transitions
 *)
 
-RegExp2NA = NA + RegExp +
+RegExp2NA = RegExp + NA +
 
 types 'a bitsNA = ('a,bool list)na