src/HOLCF/IOA/meta_theory/Abstraction.thy
changeset 23560 e43686246de4
parent 19741 f65265d71426
child 25135 4f8176c940cf
equal deleted inserted replaced
23559:0de527730294 23560:e43686246de4
     5 
     5 
     6 header {* Abstraction Theory -- tailored for I/O automata *}
     6 header {* Abstraction Theory -- tailored for I/O automata *}
     7 
     7 
     8 theory Abstraction
     8 theory Abstraction
     9 imports LiveIOA
     9 imports LiveIOA
       
    10 uses ("ioa_package.ML")
    10 begin
    11 begin
    11 
    12 
    12 defaultsort type
    13 defaultsort type
    13 
    14 
    14 consts
    15 consts
   637       auto_tac (cs addSIs weak_strength_lemmas,
   638       auto_tac (cs addSIs weak_strength_lemmas,
   638         ss addsimps [state_strengthening_def, state_weakening_def]))) i
   639         ss addsimps [state_strengthening_def, state_weakening_def]))) i
   639 end
   640 end
   640 *}
   641 *}
   641 
   642 
       
   643 use "ioa_package.ML"
       
   644 
   642 end
   645 end