src/Doc/How_to_Prove_it/How_to_Prove_it.thy
changeset 69505 cc2d676d5395
parent 67406 23307fd33906
child 69597 ff784d5a5bfb
--- a/src/Doc/How_to_Prove_it/How_to_Prove_it.thy	Wed Dec 26 16:07:28 2018 +0100
+++ b/src/Doc/How_to_Prove_it/How_to_Prove_it.thy	Wed Dec 26 16:25:20 2018 +0100
@@ -17,10 +17,10 @@
 \end{quote}
 This is often called ``complete induction''. It is applied like this:
 \begin{quote}
-(@{text"induction n rule: less_induct"})
+(\<open>induction n rule: less_induct\<close>)
 \end{quote}
 In fact, it is not restricted to @{typ nat} but works for any wellfounded
-order @{text"<"}.
+order \<open><\<close>.
 
 There are many more special induction rules. You can find all of them
 via the Find button (in Isabelle/jedit) with the following search criteria:
@@ -39,7 +39,7 @@
 lemma fixes x :: int shows "x ^ 3 = x * x * x"
 by (simp add: numeral_eq_Suc)
 
-text\<open>This is a typical situation: function ``@{text"^"}'' is defined
+text\<open>This is a typical situation: function ``\<open>^\<close>'' is defined
 by pattern matching on @{const Suc} but is applied to a numeral.
 
 Note: simplification with @{thm[source] numeral_eq_Suc} will convert all numerals.
@@ -74,8 +74,8 @@
 \section{Algebraic simplification}
 
 On the numeric types @{typ nat}, @{typ int} and @{typ real},
-proof method @{text simp} and friends can deal with a limited amount of linear
-arithmetic (no multiplication except by numerals) and method @{text arith} can
+proof method \<open>simp\<close> and friends can deal with a limited amount of linear
+arithmetic (no multiplication except by numerals) and method \<open>arith\<close> can
 handle full linear arithmetic (on @{typ nat}, @{typ int} including quantifiers).
 But what to do when proper multiplication is involved?
 At this point it can be helpful to simplify with the lemma list