src/Doc/Isar_Ref/Framework.thy
changeset 63669 256fc20716f2
parent 63531 847eefdca90d
child 63680 6e1e8b5abbfa
--- a/src/Doc/Isar_Ref/Framework.thy	Thu Aug 11 18:26:16 2016 +0200
+++ b/src/Doc/Isar_Ref/Framework.thy	Thu Aug 11 18:26:44 2016 +0200
@@ -89,7 +89,7 @@
   \<^medskip>
   Concrete applications require another intermediate layer: an object-logic.
   Isabelle/HOL @{cite "isa-tutorial"} (simply-typed set-theory) is most
-  commonly used; elementary examples are given in the directory @{file
+  commonly used; elementary examples are given in the directory @{dir
   "~~/src/HOL/Isar_Examples"}. Some examples demonstrate how to start a fresh
   object-logic from Isabelle/Pure, and use Isar proofs from the very start,
   despite the lack of advanced proof tools at such an early stage (e.g.\ see
@@ -524,7 +524,7 @@
   may be populated later. The command \<^theory_text>\<open>method_setup\<close> allows to define proof
   methods semantically in Isabelle/ML. The Eisbach language allows to define
   proof methods symbolically, as recursive expressions over existing methods
-  @{cite "Matichuk-et-al:2014"}; see also @{file "~~/src/HOL/Eisbach"}.
+  @{cite "Matichuk-et-al:2014"}; see also @{dir "~~/src/HOL/Eisbach"}.
 
   Methods use the facts indicated by \<^theory_text>\<open>then\<close> or \<^theory_text>\<open>using\<close>, and then operate on
   the goal state. Some basic methods are predefined in Pure: ``@{method "-"}''