# HG changeset patch # User wenzelm # Date 1632250566 -7200 # Node ID e5ff77db6f386bb6d8f2189f6e6ebd58f3655e98 # Parent 1c2c0380d58b7881919be494c165a7807c35e043 clarified antiquotations; diff -r 1c2c0380d58b -r e5ff77db6f38 src/HOL/Transitive_Closure.thy --- a/src/HOL/Transitive_Closure.thy Tue Sep 21 19:42:30 2021 +0200 +++ b/src/HOL/Transitive_Closure.thy Tue Sep 21 20:56:06 2021 +0200 @@ -1287,12 +1287,12 @@ val trancl_rtrancl_trancl = @{thm trancl_rtrancl_trancl}; val rtrancl_trans = @{thm rtrancl_trans}; - fun decomp (\<^const>\Trueprop\ $ t) = + fun decomp \<^Const_>\Trueprop for t\ = let - fun dec (Const (\<^const_name>\Set.member\, _) $ (Const (\<^const_name>\Pair\, _) $ a $ b) $ rel) = + fun dec \<^Const_>\Set.member _ for \\<^Const_>\Pair _ _ for a b\\ rel\ = let - fun decr (Const (\<^const_name>\rtrancl\, _ ) $ r) = (r,"r*") - | decr (Const (\<^const_name>\trancl\, _ ) $ r) = (r,"r+") + fun decr \<^Const_>\rtrancl _ for r\ = (r,"r*") + | decr \<^Const_>\trancl _ for r\ = (r,"r+") | decr r = (r,"r"); val (rel,r) = decr (Envir.beta_eta_contract rel); in SOME (a,b,rel,r) end @@ -1312,12 +1312,12 @@ val trancl_rtrancl_trancl = @{thm tranclp_rtranclp_tranclp}; val rtrancl_trans = @{thm rtranclp_trans}; - fun decomp (\<^const>\Trueprop\ $ t) = + fun decomp \<^Const_>\Trueprop for t\ = let fun dec (rel $ a $ b) = let - fun decr (Const (\<^const_name>\rtranclp\, _ ) $ r) = (r,"r*") - | decr (Const (\<^const_name>\tranclp\, _ ) $ r) = (r,"r+") + fun decr \<^Const_>\rtranclp _ for r\ = (r,"r*") + | decr \<^Const_>\tranclp _ for r\ = (r,"r+") | decr r = (r,"r"); val (rel,r) = decr rel; in SOME (a, b, rel, r) end diff -r 1c2c0380d58b -r e5ff77db6f38 src/HOL/Typerep.thy --- a/src/HOL/Typerep.thy Tue Sep 21 19:42:30 2021 +0200 +++ b/src/HOL/Typerep.thy Tue Sep 21 20:56:06 2021 +0200 @@ -32,8 +32,7 @@ typed_print_translation \ let - fun typerep_tr' ctxt (*"typerep"*) - (Type (\<^type_name>\fun\, [Type (\<^type_name>\itself\, [T]), _])) + fun typerep_tr' ctxt (*"typerep"*) \<^Type>\fun \\<^Type>\itself T\\ _\ (Const (\<^const_syntax>\Pure.type\, _) :: ts) = Term.list_comb (Syntax.const \<^syntax_const>\_TYPEREP\ $ Syntax_Phases.term_of_typ ctxt T, ts) @@ -49,10 +48,9 @@ val sorts = replicate (Sign.arity_number thy tyco) \<^sort>\typerep\; val vs = Name.invent_names Name.context "'a" sorts; val ty = Type (tyco, map TFree vs); - val lhs = Const (\<^const_name>\typerep\, Term.itselfT ty --> \<^typ>\typerep\) - $ Free ("T", Term.itselfT ty); - val rhs = \<^term>\Typerep\ $ HOLogic.mk_literal tyco - $ HOLogic.mk_list \<^typ>\typerep\ (map (HOLogic.mk_typerep o TFree) vs); + val lhs = \<^Const>\typerep ty\ $ Free ("T", Term.itselfT ty); + val rhs = \<^Const>\Typerep\ $ HOLogic.mk_literal tyco + $ HOLogic.mk_list \<^Type>\typerep\ (map (HOLogic.mk_typerep o TFree) vs); val eq = HOLogic.mk_Trueprop (HOLogic.mk_eq (lhs, rhs)); in thy