src/HOL/FunDef.thy
changeset 29127 2a684ee023e7
parent 29125 d41182a8135c
child 29580 117b88da143c
--- a/src/HOL/FunDef.thy	Tue Dec 16 18:04:31 2008 +0100
+++ b/src/HOL/FunDef.thy	Tue Dec 16 19:24:55 2008 +0100
@@ -235,7 +235,7 @@
 lemma wf_pair_less[simp]: "wf pair_less"
   by (auto simp: pair_less_def)
 
-text {* Introduction rules for pair_less/pair_leq *}
+text {* Introduction rules for @{text pair_less}/@{text pair_leq} *}
 lemma pair_leqI1: "a < b \<Longrightarrow> ((a, s), (b, t)) \<in> pair_leq"
   and pair_leqI2: "a \<le> b \<Longrightarrow> s \<le> t \<Longrightarrow> ((a, s), (b, t)) \<in> pair_leq"
   and pair_lessI1: "a < b  \<Longrightarrow> ((a, s), (b, t)) \<in> pair_less"