src/Doc/Codegen/Introduction.thy
changeset 72375 e48d93811ed7
parent 70011 9dde788b0128
child 76649 9a6cb5ecc183
--- a/src/Doc/Codegen/Introduction.thy	Sat Oct 03 23:01:40 2020 +0100
+++ b/src/Doc/Codegen/Introduction.thy	Mon Oct 05 21:15:58 2020 +0200
@@ -3,7 +3,7 @@
 begin (*<*)
 
 ML \<open>
-  Isabelle_System.mkdirs (File.tmp_path (Path.basic "examples"))
+  Isabelle_System.make_directory (File.tmp_path (Path.basic "examples"))
 \<close> (*>*)
 
 section \<open>Introduction\<close>