src/HOL/Decision_Procs/Approximation.thy
changeset 69605 a96320074298
parent 69597 ff784d5a5bfb
child 69830 54d19f1f0ba6
--- a/src/HOL/Decision_Procs/Approximation.thy	Sun Jan 06 13:44:33 2019 +0100
+++ b/src/HOL/Decision_Procs/Approximation.thy	Sun Jan 06 15:04:34 2019 +0100
@@ -1635,7 +1635,7 @@
   "n \<in> {m .. l} \<longleftrightarrow> real n \<in> {real m .. real l}"
   by (simp_all add: real_div_nat_eq_floor_of_divide minus_div_mult_eq_mod [symmetric])
 
-ML_file "approximation.ML"
+ML_file \<open>approximation.ML\<close>
 
 method_setup approximation = \<open>
   let
@@ -1667,7 +1667,7 @@
     "\<not> \<not> q \<longleftrightarrow> q"
   by auto
 
-ML_file "approximation_generator.ML"
+ML_file \<open>approximation_generator.ML\<close>
 setup "Approximation_Generator.setup"
 
 end