--- a/src/HOL/Matrix_LP/ComputeFloat.thy Sun Jan 06 13:44:33 2019 +0100
+++ b/src/HOL/Matrix_LP/ComputeFloat.thy Sun Jan 06 15:04:34 2019 +0100
@@ -8,7 +8,7 @@
imports Complex_Main "HOL-Library.Lattice_Algebras"
begin
-ML_file "~~/src/Tools/float.ML"
+ML_file \<open>~~/src/Tools/float.ML\<close>
(*FIXME surely floor should be used? This file is full of redundant material.*)
@@ -235,6 +235,6 @@
lemmas arith = arith_simps rel_simps diff_nat_numeral nat_0
nat_neg_numeral powerarith floatarith not_false_eq_true not_true_eq_false
-ML_file "float_arith.ML"
+ML_file \<open>float_arith.ML\<close>
end