new style theory
authornipkow
Thu, 17 Jan 2002 19:37:57 +0100
changeset 12794 c992ee4168ff
parent 12793 e99d4a6cba8b
child 12795 fc716621f19d
new style theory
src/HOL/Lex/Scanner.ML
--- a/src/HOL/Lex/Scanner.ML	Thu Jan 17 19:37:42 2002 +0100
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,15 +0,0 @@
-(*  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";