diff -r a80d8ec6c998 -r 3dda49e08b9d src/HOL/Inductive.thy --- a/src/HOL/Inductive.thy Fri Jan 04 21:49:06 2019 +0100 +++ b/src/HOL/Inductive.thy Fri Jan 04 23:22:53 2019 +0100 @@ -270,8 +270,8 @@ subsection \Even Stronger Coinduction Rule, by Martin Coen\ -text \Weakens the condition @{term "X \ f X"} to one expressed using both - @{term lfp} and @{term gfp}\ +text \Weakens the condition \<^term>\X \ f X\ to one expressed using both + \<^term>\lfp\ and \<^term>\gfp\\ lemma coinduct3_mono_lemma: "mono f \ mono (\x. f x \ X \ B)" by (iprover intro: subset_refl monoI Un_mono monoD) @@ -312,7 +312,7 @@ lemma def_coinduct3: "A \ gfp f \ mono f \ a \ X \ X \ f (lfp (\x. f x \ X \ A)) \ a \ A" by (auto intro!: coinduct3) -text \Monotonicity of @{term gfp}!\ +text \Monotonicity of \<^term>\gfp\!\ lemma gfp_mono: "(\Z. f Z \ g Z) \ gfp f \ gfp g" by (rule gfp_upperbound [THEN gfp_least]) (blast intro: order_trans) @@ -535,7 +535,7 @@ val x = Syntax.free (fst (Name.variant "x" (Term.declare_term_frees cs Name.context))); val ft = Case_Translation.case_tr true ctxt [x, cs]; in lambda x ft end - in [(@{syntax_const "_lam_pats_syntax"}, fun_tr)] end + in [(\<^syntax_const>\_lam_pats_syntax\, fun_tr)] end \ end