src/HOL/Library/Phantom_Type.thy
changeset 60500 903bb1495239
parent 58881 b9556a055632
child 69593 3dda49e08b9d
--- a/src/HOL/Library/Phantom_Type.thy	Wed Jun 17 10:57:11 2015 +0200
+++ b/src/HOL/Library/Phantom_Type.thy	Wed Jun 17 11:03:05 2015 +0200
@@ -2,7 +2,7 @@
     Author:     Andreas Lochbihler
 *)
 
-section {* A generic phantom type *}
+section \<open>A generic phantom type\<close>
 
 theory Phantom_Type
 imports Main
@@ -21,14 +21,14 @@
 translations
   "Phantom('t)" => "CONST phantom :: _ \<Rightarrow> ('t, _) phantom"
 
-typed_print_translation {*
+typed_print_translation \<open>
   let
     fun phantom_tr' ctxt (Type (@{type_name fun}, [_, Type (@{type_name phantom}, [T, _])])) ts =
           list_comb
             (Syntax.const @{syntax_const "_Phantom"} $ Syntax_Phases.term_of_typ ctxt T, ts)
       | phantom_tr' _ _ _ = raise Match;
   in [(@{const_syntax phantom}, phantom_tr')] end
-*}
+\<close>
 
 lemma of_phantom_inject [simp]:
   "of_phantom x = of_phantom y \<longleftrightarrow> x = y"