diff -r a80d8ec6c998 -r 3dda49e08b9d src/HOL/Library/Countable.thy --- a/src/HOL/Library/Countable.thy Fri Jan 04 21:49:06 2019 +0100 +++ b/src/HOL/Library/Countable.thy Fri Jan 04 23:22:53 2019 +0100 @@ -168,7 +168,7 @@ let val ty_name = (case goal of - (_ $ Const (@{const_name Pure.type}, Type (@{type_name itself}, [Type (n, _)]))) => n + (_ $ Const (\<^const_name>\Pure.type\, Type (\<^type_name>\itself\, [Type (n, _)]))) => n | _ => raise Match) val typedef_info = hd (Typedef.get_info ctxt ty_name) val typedef_thm = #type_definition (snd typedef_info) @@ -183,7 +183,7 @@ val induct_thm = the (AList.lookup (op =) alist pred_name) val vars = rev (Term.add_vars (Thm.prop_of induct_thm) []) val insts = vars |> map (fn (_, T) => try (Thm.cterm_of ctxt) - (Const (@{const_name Countable.finite_item}, T))) + (Const (\<^const_name>\Countable.finite_item\, T))) val induct_thm' = Thm.instantiate' [] insts induct_thm val rules = @{thms finite_item.intros} in