src/Doc/Main/Main_Doc.thy
changeset 65964 3de7464450b0
parent 65956 639eb3617a86
child 66435 292680dde314
equal deleted inserted replaced
65963:ca1e636fa716 65964:3de7464450b0
    59 
    59 
    60 \begin{supertabular}{@ {} l @ {~::~} l l @ {}}
    60 \begin{supertabular}{@ {} l @ {~::~} l l @ {}}
    61 @{const Orderings.less_eq} & @{typeof Orderings.less_eq} & (\<^verbatim>\<open><=\<close>)\\
    61 @{const Orderings.less_eq} & @{typeof Orderings.less_eq} & (\<^verbatim>\<open><=\<close>)\\
    62 @{const Orderings.less} & @{typeof Orderings.less}\\
    62 @{const Orderings.less} & @{typeof Orderings.less}\\
    63 @{const Orderings.Least} & @{typeof Orderings.Least}\\
    63 @{const Orderings.Least} & @{typeof Orderings.Least}\\
       
    64 @{const Orderings.Greatest} & @{typeof Orderings.Greatest}\\
    64 @{const Orderings.min} & @{typeof Orderings.min}\\
    65 @{const Orderings.min} & @{typeof Orderings.min}\\
    65 @{const Orderings.max} & @{typeof Orderings.max}\\
    66 @{const Orderings.max} & @{typeof Orderings.max}\\
    66 @{const Lattices_Big.arg_min} & @{typeof Lattices_Big.arg_min}\\
       
    67 @{const[source] top} & @{typeof Orderings.top}\\
    67 @{const[source] top} & @{typeof Orderings.top}\\
    68 @{const[source] bot} & @{typeof Orderings.bot}\\
    68 @{const[source] bot} & @{typeof Orderings.bot}\\
    69 @{const Orderings.mono} & @{typeof Orderings.mono}\\
    69 @{const Orderings.mono} & @{typeof Orderings.mono}\\
    70 @{const Orderings.strict_mono} & @{typeof Orderings.strict_mono}\\
    70 @{const Orderings.strict_mono} & @{typeof Orderings.strict_mono}\\
    71 \end{supertabular}
    71 \end{supertabular}
    77 @{term[source]"x > y"} & @{term"x > y"}\\
    77 @{term[source]"x > y"} & @{term"x > y"}\\
    78 @{term "\<forall>x\<le>y. P"} & @{term[source]"\<forall>x. x \<le> y \<longrightarrow> P"}\\
    78 @{term "\<forall>x\<le>y. P"} & @{term[source]"\<forall>x. x \<le> y \<longrightarrow> P"}\\
    79 @{term "\<exists>x\<le>y. P"} & @{term[source]"\<exists>x. x \<le> y \<and> P"}\\
    79 @{term "\<exists>x\<le>y. P"} & @{term[source]"\<exists>x. x \<le> y \<and> P"}\\
    80 \multicolumn{2}{@ {}l@ {}}{Similarly for $<$, $\ge$ and $>$}\\
    80 \multicolumn{2}{@ {}l@ {}}{Similarly for $<$, $\ge$ and $>$}\\
    81 @{term "LEAST x. P"} & @{term[source]"Least (\<lambda>x. P)"}\\
    81 @{term "LEAST x. P"} & @{term[source]"Least (\<lambda>x. P)"}\\
       
    82 @{term "GREATEST x. P"} & @{term[source]"Greatest (\<lambda>x. P)"}\\
    82 \end{supertabular}
    83 \end{supertabular}
    83 
    84 
    84 
    85 
    85 \section*{Lattices}
    86 \section*{Lattices}
    86 
    87 
   418 @{const Lattices_Big.Max} & @{typeof Lattices_Big.Max}\\
   419 @{const Lattices_Big.Max} & @{typeof Lattices_Big.Max}\\
   419 @{const Lattices_Big.arg_min} & @{typeof Lattices_Big.arg_min}\\
   420 @{const Lattices_Big.arg_min} & @{typeof Lattices_Big.arg_min}\\
   420 @{const Lattices_Big.is_arg_min} & @{typeof Lattices_Big.is_arg_min}\\
   421 @{const Lattices_Big.is_arg_min} & @{typeof Lattices_Big.is_arg_min}\\
   421 @{const Lattices_Big.arg_max} & @{typeof Lattices_Big.arg_max}\\
   422 @{const Lattices_Big.arg_max} & @{typeof Lattices_Big.arg_max}\\
   422 @{const Lattices_Big.is_arg_max} & @{typeof Lattices_Big.is_arg_max}\\
   423 @{const Lattices_Big.is_arg_max} & @{typeof Lattices_Big.is_arg_max}\\
   423 @{const Lattices_Big.Greatest} & @{typeof Lattices_Big.Greatest}\\
       
   424 \end{supertabular}
   424 \end{supertabular}
   425 
   425 
   426 \subsubsection*{Syntax}
   426 \subsubsection*{Syntax}
   427 
   427 
   428 \begin{supertabular}{@ {} l @ {\quad$\equiv$\quad} l l @ {}}
   428 \begin{supertabular}{@ {} l @ {\quad$\equiv$\quad} l l @ {}}
   429 @{term "ARG_MIN f x. P"} & @{term[source]"arg_min f (\<lambda>x. P)"}\\
   429 @{term "ARG_MIN f x. P"} & @{term[source]"arg_min f (\<lambda>x. P)"}\\
   430 @{term "ARG_MAX f x. P"} & @{term[source]"arg_max f (\<lambda>x. P)"}\\
   430 @{term "ARG_MAX f x. P"} & @{term[source]"arg_max f (\<lambda>x. P)"}\\
   431 @{term "GREATEST x. P"} & @{term[source]"Greatest (\<lambda>x. P)"}\\
       
   432 \end{supertabular}
   431 \end{supertabular}
   433 
   432 
   434 
   433 
   435 \section*{Groups\_Big}
   434 \section*{Groups\_Big}
   436 
   435