doc-src/Main/Docs/Main_Doc.thy
changeset 47189 e9a3dd1c4cf9
parent 47187 97db4b6b6a2c
child 47682 8e2e87a0a594
equal deleted inserted replaced
47188:da9a2d9e1143 47189:e9a3dd1c4cf9
    14       (Args.term -- Args.typ_abbrev)
    14       (Args.term -- Args.typ_abbrev)
    15       (fn {source, context = ctxt, ...} => fn arg =>
    15       (fn {source, context = ctxt, ...} => fn arg =>
    16         Thy_Output.output ctxt
    16         Thy_Output.output ctxt
    17           (Thy_Output.maybe_pretty_source pretty_term_type_only ctxt source [arg]))
    17           (Thy_Output.maybe_pretty_source pretty_term_type_only ctxt source [arg]))
    18   end
    18   end
       
    19 *}
       
    20 setup {*
       
    21   Thy_Output.antiquotation @{binding expanded_typ} (Args.typ >> single)
       
    22     (fn {source, context, ...} => Thy_Output.output context o
       
    23       Thy_Output.maybe_pretty_source Syntax.pretty_typ context source)
    19 *}
    24 *}
    20 (*>*)
    25 (*>*)
    21 text{*
    26 text{*
    22 
    27 
    23 \begin{abstract}
    28 \begin{abstract}
   262 @{term"converse r"} & @{term[source]"converse r"} & (\verb$^-1$)
   267 @{term"converse r"} & @{term[source]"converse r"} & (\verb$^-1$)
   263 \end{tabular}
   268 \end{tabular}
   264 \medskip
   269 \medskip
   265 
   270 
   266 \noindent
   271 \noindent
   267 Type synonym @{typ"'a rel"} @{text"="} @{typ "('a * 'a)set"}
   272 Type synonym \ @{typ"'a rel"} @{text"="} @{expanded_typ "'a rel"}
   268 
   273 
   269 \section{Equiv\_Relations}
   274 \section{Equiv\_Relations}
   270 
   275 
   271 \begin{supertabular}{@ {} l @ {~::~} l @ {}}
   276 \begin{supertabular}{@ {} l @ {~::~} l @ {}}
   272 @{const Equiv_Relations.equiv} & @{term_type_only Equiv_Relations.equiv "'a set \<Rightarrow> ('a*'a)set\<Rightarrow>bool"}\\
   277 @{const Equiv_Relations.equiv} & @{term_type_only Equiv_Relations.equiv "'a set \<Rightarrow> ('a*'a)set\<Rightarrow>bool"}\\