src/HOL/Lex/Auto.thy
changeset 1374 5e407f2a3323
parent 1344 f172a7f14e49
child 1476 608483c2122a
--- a/src/HOL/Lex/Auto.thy	Wed Nov 29 16:58:30 1995 +0100
+++ b/src/HOL/Lex/Auto.thy	Wed Nov 29 17:01:41 1995 +0100
@@ -17,12 +17,12 @@
 types ('a,'b)auto = "'b * ('b => 'a => 'b) * ('b => bool)"
 
 consts
-  start :: "('a, 'b)auto => 'b"
-  next  :: "('a, 'b)auto => ('b => 'a => 'b)"
-  fin   :: "('a, 'b)auto => ('b => bool)"
-  nexts :: "('a, 'b)auto => 'b => 'a list => 'b"
-  accepts :: "('a,'b) auto => 'a list => bool"  
-  acc_prefix :: "('a, 'b)auto => 'b => 'a list => bool"
+  start :: ('a, 'b)auto => 'b
+  next  :: ('a, 'b)auto => ('b => 'a => 'b)
+  fin   :: ('a, 'b)auto => ('b => bool)
+  nexts :: ('a, 'b)auto => 'b => 'a list => 'b
+  accepts :: ('a,'b) auto => 'a list => bool  
+  acc_prefix :: ('a, 'b)auto => 'b => 'a list => bool
 
 defs
   start_def "start(A) == fst(A)"