src/HOL/Lex/Scanner.ML
author oheimb
Thu, 01 Feb 2001 20:51:48 +0100
changeset 11025 a70b796d9af8
parent 5323 028e00595280
permissions -rw-r--r--
converted to Isar therory, adding attributes complete_split and split_format

(*  Title:      HOL/Lex/Scanner.ML
    ID:         $Id$
    Author:     Tobias Nipkow
    Copyright   1998 TUM
*)

Goal
 "DA.accepts (na2da(rexp2na r)) w = (w : lang r)";
by (simp_tac (simpset() addsimps [NA_DA_equiv RS sym,accepts_rexp2na]) 1);
qed "accepts_na2da_rexp2na";

Goal
 "DA.accepts (nae2da(rexp2nae r)) w = (w : lang r)";
by (simp_tac (simpset() addsimps [NAe_DA_equiv,accepts_rexp2nae]) 1);
qed "accepts_nae2da_rexp2nae";