src/HOL/Isar_examples/Group.thy
changeset 7761 7fab9592384f
parent 7748 5b9c45b21782
child 7800 8ee919e42174
equal deleted inserted replaced
7760:43f8d28dbc6e 7761:7fab9592384f
    69     by (simp only: group_left_unit);
    69     by (simp only: group_left_unit);
    70   finally; show ?thesis; .;
    70   finally; show ?thesis; .;
    71 qed;
    71 qed;
    72 
    72 
    73 text {*
    73 text {*
    74  There are only two Isar language elements for calculational proofs:
    74  \bigskip There are only two Isar language elements for calculational
    75  \isakeyword{also} for initial or intermediate calculational steps,
    75  proofs: \isakeyword{also} for initial or intermediate calculational
    76  and \isakeyword{finally} for building the result of a calculation.
    76  steps, and \isakeyword{finally} for building the result of a
    77  These constructs are not hardwired into Isabelle/Isar, but defined on
    77  calculation.  These constructs are not hardwired into Isabelle/Isar,
    78  top of the basic Isar/VM interpreter.  Expanding the
    78  but defined on top of the basic Isar/VM interpreter.  Expanding the
    79  \isakeyword{also} and \isakeyword{finally} derived language elements,
    79  \isakeyword{also} and \isakeyword{finally} derived language elements,
    80  calculations may be simulated as demonstrated below.
    80  calculations may be simulated as demonstrated below.
    81 
    81 
    82  Note that ``$\dots$'' is just a special term binding that happens to
    82  Note that ``$\dots$'' is just a special term binding that happens to
    83  be bound automatically to the argument of the last fact established
    83  be bound automatically to the argument of the last fact established
   115 
   115 
   116   show ?thesis; .;
   116   show ?thesis; .;
   117 qed;
   117 qed;
   118 
   118 
   119 
   119 
   120 subsection {* Groups and monoids *};
   120 subsection {* Groups as monoids *};
   121 
   121 
   122 text {*
   122 text {*
   123   Monoids are usually defined like this.
   123   Monoids are usually defined like this.
   124 *};
   124 *};
   125 
   125