src/HOL/Partial_Function.thy
changeset 69605 a96320074298
parent 69593 3dda49e08b9d
child 69745 aec42cee2521
--- a/src/HOL/Partial_Function.thy	Sun Jan 06 13:44:33 2019 +0100
+++ b/src/HOL/Partial_Function.thy	Sun Jan 06 15:04:34 2019 +0100
@@ -10,7 +10,7 @@
 begin
 
 named_theorems partial_function_mono "monotonicity rules for partial function definitions"
-ML_file "Tools/Function/partial_function.ML"
+ML_file \<open>Tools/Function/partial_function.ML\<close>
 
 lemma (in ccpo) in_chain_finite:
   assumes "Complete_Partial_Order.chain (\<le>) A" "finite A" "A \<noteq> {}"