doc-src/TutorialI/Types/Axioms.thy
changeset 10420 ef006735bee8
parent 10396 5ab08609e6c8
child 10654 458068404143
equal deleted inserted replaced
10419:1bfdd19c1d47 10420:ef006735bee8
    26 The first three axioms are the familiar ones, and the final one
    26 The first three axioms are the familiar ones, and the final one
    27 requires that @{text"<<"} and @{text"<<="} are related as expected.
    27 requires that @{text"<<"} and @{text"<<="} are related as expected.
    28 Note that behind the scenes, Isabelle has restricted the axioms to class
    28 Note that behind the scenes, Isabelle has restricted the axioms to class
    29 @{text parord}. For example, this is what @{thm[source]refl} really looks like:
    29 @{text parord}. For example, this is what @{thm[source]refl} really looks like:
    30 @{thm[show_types]refl}.
    30 @{thm[show_types]refl}.
       
    31 
       
    32 We have not made @{thm[source]less_le} a global definition because it would
       
    33 fix once and for all that @{text"<<"} is defined in terms of @{text"<<="}.
       
    34 There are however situations where it is the other way around, which such a
       
    35 definition would complicate. The slight drawback of the above class is that
       
    36 we need to define both @{text"<<="} and @{text"<<"} for each instance.
    31 
    37 
    32 We can now prove simple theorems in this abstract setting, for example
    38 We can now prove simple theorems in this abstract setting, for example
    33 that @{text"<<"} is not symmetric:
    39 that @{text"<<"} is not symmetric:
    34 *}
    40 *}
    35 
    41