src/HOLCF/IOA/meta_theory/Abstraction.thy
changeset 31773 4d33c5d7575b
parent 31738 7b9b9ba532ca
child 32149 ef59550a55d3
--- 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