src/HOL/HOLCF/Domain_Aux.thy
changeset 69605 a96320074298
parent 68383 93a42bd62ede
child 78793 2cb027b95188
equal deleted inserted replaced
69604:d80b2df54d31 69605:a96320074298
   353 subsection \<open>ML setup\<close>
   353 subsection \<open>ML setup\<close>
   354 
   354 
   355 named_theorems domain_deflation "theorems like deflation a ==> deflation (foo_map$a)"
   355 named_theorems domain_deflation "theorems like deflation a ==> deflation (foo_map$a)"
   356   and domain_map_ID "theorems like foo_map$ID = ID"
   356   and domain_map_ID "theorems like foo_map$ID = ID"
   357 
   357 
   358 ML_file "Tools/Domain/domain_take_proofs.ML"
   358 ML_file \<open>Tools/Domain/domain_take_proofs.ML\<close>
   359 ML_file "Tools/cont_consts.ML"
   359 ML_file \<open>Tools/cont_consts.ML\<close>
   360 ML_file "Tools/cont_proc.ML"
   360 ML_file \<open>Tools/cont_proc.ML\<close>
   361 ML_file "Tools/Domain/domain_constructors.ML"
   361 ML_file \<open>Tools/Domain/domain_constructors.ML\<close>
   362 ML_file "Tools/Domain/domain_induction.ML"
   362 ML_file \<open>Tools/Domain/domain_induction.ML\<close>
   363 
   363 
   364 end
   364 end