renamed ioa to automaton
authorhaftmann
Tue, 23 Jun 2009 12:08:35 +0200
changeset 31773 4d33c5d7575b
parent 31772 a946fe9a0476
child 31774 5c8cfaed32e6
renamed ioa to automaton
src/HOLCF/IOA/meta_theory/Abstraction.thy
src/HOLCF/IsaMakefile
--- a/src/HOLCF/IOA/meta_theory/Abstraction.thy	Tue Jun 23 12:08:34 2009 +0200
+++ b/src/HOLCF/IOA/meta_theory/Abstraction.thy	Tue Jun 23 12:08:35 2009 +0200
@@ -6,7 +6,7 @@
 
 theory Abstraction
 imports LiveIOA
-uses ("ioa.ML")
+uses ("automaton.ML")
 begin
 
 defaultsort type
@@ -613,6 +613,6 @@
 
 method_setup abstraction = {* Scan.succeed (SIMPLE_METHOD' o abstraction_tac) *} ""
 
-use "ioa.ML"
+use "automaton.ML"
 
 end
--- a/src/HOLCF/IsaMakefile	Tue Jun 23 12:08:34 2009 +0200
+++ b/src/HOLCF/IsaMakefile	Tue Jun 23 12:08:35 2009 +0200
@@ -127,7 +127,7 @@
   IOA/meta_theory/TL.thy IOA/meta_theory/TLS.thy		       \
   IOA/meta_theory/LiveIOA.thy IOA/meta_theory/Pred.thy		       \
   IOA/meta_theory/Abstraction.thy IOA/meta_theory/Simulations.thy      \
-  IOA/meta_theory/SimCorrectness.thy IOA/meta_theory/ioa.ML
+  IOA/meta_theory/SimCorrectness.thy IOA/meta_theory/automaton.ML
 	@cd IOA; $(ISABELLE_TOOL) usedir -b $(OUT)/HOLCF IOA