src/HOL/Lex/Scanner.ML
author wenzelm
Mon, 22 Jun 1998 17:26:46 +0200
changeset 5069 3ea049f7979d
parent 4907 0eb6730de30f
child 5132 24f992a25adc
permissions -rw-r--r--
isatool fixgoal;
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.ML
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
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4907
diff changeset
     7
Goal
4907
0eb6730de30f Reshuffeling, renaming and a few simple corollaries.
nipkow
parents:
diff changeset
     8
 "DA.accepts (nae2da(rexp2nae r)) w = (w : lang r)";
0eb6730de30f Reshuffeling, renaming and a few simple corollaries.
nipkow
parents:
diff changeset
     9
by(simp_tac (simpset() addsimps [NAe_DA_equiv,accepts_rexp2nae]) 1);
0eb6730de30f Reshuffeling, renaming and a few simple corollaries.
nipkow
parents:
diff changeset
    10
qed "accepts_nae2da_rexp2nae";