src/HOL/Lex/Scanner.thy
author paulson
Wed, 05 Aug 1998 10:57:25 +0200
changeset 5253 82a5ca6290aa
parent 4907 0eb6730de30f
child 5323 028e00595280
permissions -rw-r--r--
New record type of programs
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
4907
0eb6730de30f Reshuffeling, renaming and a few simple corollaries.
nipkow
parents:
diff changeset
     1
(*  Title:      HOL/Lex/Scanner.thy
0eb6730de30f Reshuffeling, renaming and a few simple corollaries.
nipkow
parents:
diff changeset
     2
    ID:         $Id$
0eb6730de30f Reshuffeling, renaming and a few simple corollaries.
nipkow
parents:
diff changeset
     3
    Author:     Tobias Nipkow
0eb6730de30f Reshuffeling, renaming and a few simple corollaries.
nipkow
parents:
diff changeset
     4
    Copyright   1998 TUM
0eb6730de30f Reshuffeling, renaming and a few simple corollaries.
nipkow
parents:
diff changeset
     5
*)
0eb6730de30f Reshuffeling, renaming and a few simple corollaries.
nipkow
parents:
diff changeset
     6
0eb6730de30f Reshuffeling, renaming and a few simple corollaries.
nipkow
parents:
diff changeset
     7
Scanner = Automata + RegExp2NAe