doc-src/TutorialI/Sets/sets.tex
changeset 30649 57753e0ec1d4
parent 25341 ca3761e38a87
child 42637 381fdcab0f36
equal deleted inserted replaced
30617:620db300c038 30649:57753e0ec1d4
   297 Unions can be formed over the values of a given  set.  The syntax is
   297 Unions can be formed over the values of a given  set.  The syntax is
   298 \mbox{\isa{\isasymUnion x\isasymin A.\ B}} or 
   298 \mbox{\isa{\isasymUnion x\isasymin A.\ B}} or 
   299 \isa{UN x:A.\ B} in \textsc{ascii}. Indexed union satisfies this basic law:
   299 \isa{UN x:A.\ B} in \textsc{ascii}. Indexed union satisfies this basic law:
   300 \begin{isabelle}
   300 \begin{isabelle}
   301 (b\ \isasymin\
   301 (b\ \isasymin\
   302 (\isasymUnion x\isasymin A. B\ x) =\ (\isasymexists x\isasymin A.\
   302 (\isasymUnion x\isasymin A. B\ x)) =\ (\isasymexists x\isasymin A.\
   303 b\ \isasymin\ B\ x)
   303 b\ \isasymin\ B\ x)
   304 \rulenamedx{UN_iff}
   304 \rulenamedx{UN_iff}
   305 \end{isabelle}
   305 \end{isabelle}
   306 It has two natural deduction rules similar to those for the existential
   306 It has two natural deduction rules similar to those for the existential
   307 quantifier.  Sometimes \isa{UN_I} must be applied explicitly:
   307 quantifier.  Sometimes \isa{UN_I} must be applied explicitly:
   412 \end{isabelle}
   412 \end{isabelle}
   413 Writing $|A|$ as $n$, the last of these theorems says that the number of
   413 Writing $|A|$ as $n$, the last of these theorems says that the number of
   414 $k$-element subsets of~$A$ is \index{binomial coefficients}
   414 $k$-element subsets of~$A$ is \index{binomial coefficients}
   415 $\binom{n}{k}$.
   415 $\binom{n}{k}$.
   416 
   416 
   417 \begin{warn}
   417 %\begin{warn}
   418 The term \isa{finite\ A} is defined via a syntax translation as an
   418 %The term \isa{finite\ A} is defined via a syntax translation as an
   419 abbreviation for \isa{A {\isasymin} Finites}, where the constant
   419 %abbreviation for \isa{A {\isasymin} Finites}, where the constant
   420 \cdx{Finites} denotes the set of all finite sets of a given type.  There
   420 %\cdx{Finites} denotes the set of all finite sets of a given type.  There
   421 is no constant \isa{finite}.
   421 %is no constant \isa{finite}.
   422 \end{warn}
   422 %\end{warn}
   423 \index{sets|)}
   423 \index{sets|)}
   424 
   424 
   425 
   425 
   426 \section{Functions}
   426 \section{Functions}
   427 
   427