src/HOL/Ctr_Sugar.thy
changeset 54701 4ed7454aebde
parent 54626 8a5e82425e55
child 55160 2d69438b1b0c
--- a/src/HOL/Ctr_Sugar.thy	Mon Dec 09 06:33:46 2013 +0100
+++ b/src/HOL/Ctr_Sugar.thy	Mon Dec 09 09:44:57 2013 +0100
@@ -25,7 +25,7 @@
 declare [[coercion_args case_abs -]]
 declare [[coercion_args case_elem - +]]
 
-ML_file "Tools/case_translation.ML"
+ML_file "Tools/Ctr_Sugar/case_translation.ML"
 setup Case_Translation.setup
 
 lemma iffI_np: "\<lbrakk>x \<Longrightarrow> \<not> y; \<not> x \<Longrightarrow> y\<rbrakk> \<Longrightarrow> \<not> x \<longleftrightarrow> y"
@@ -36,9 +36,9 @@
 "\<not> Q \<Longrightarrow> P \<longleftrightarrow> Q \<Longrightarrow> P \<Longrightarrow> R"
 by blast+
 
-ML_file "Tools/ctr_sugar_util.ML"
-ML_file "Tools/ctr_sugar_tactics.ML"
-ML_file "Tools/ctr_sugar_code.ML"
-ML_file "Tools/ctr_sugar.ML"
+ML_file "Tools/Ctr_Sugar/ctr_sugar_util.ML"
+ML_file "Tools/Ctr_Sugar/ctr_sugar_tactics.ML"
+ML_file "Tools/Ctr_Sugar/ctr_sugar_code.ML"
+ML_file "Tools/Ctr_Sugar/ctr_sugar.ML"
 
 end