src/HOL/Ring_and_Field.thy
changeset 14569 78b75a9eec01
parent 14504 7a3d80e276d4
child 14603 985eb6708207
equal deleted inserted replaced
14568:1acde8c39179 14569:78b75a9eec01
     3     Author:  Gertrud Bauer and Markus Wenzel, TU Muenchen
     3     Author:  Gertrud Bauer and Markus Wenzel, TU Muenchen
     4              Lawrence C Paulson, University of Cambridge
     4              Lawrence C Paulson, University of Cambridge
     5     License: GPL (GNU GENERAL PUBLIC LICENSE)
     5     License: GPL (GNU GENERAL PUBLIC LICENSE)
     6 *)
     6 *)
     7 
     7 
     8 header {*
     8 header {* Ring and field structures *}
     9   \title{Ring and field structures}
       
    10   \author{Gertrud Bauer, L. C. Paulson and Markus Wenzel}
       
    11 *}
       
    12 
     9 
    13 theory Ring_and_Field = Inductive:
    10 theory Ring_and_Field = Inductive:
    14 
    11 
    15 subsection {* Abstract algebraic structures *}
    12 subsection {* Abstract algebraic structures *}
    16 
    13