src/HOL/Algebra/abstract/Ring2.thy
changeset 22808 a7daa74e2980
parent 22384 33a46e6c7f04
child 22997 d4f3b015b50b
equal deleted inserted replaced
22807:715d01b34abb 22808:a7daa74e2980
    13 section {* Constants *}
    13 section {* Constants *}
    14 
    14 
    15 text {* Most constants are already declared by HOL. *}
    15 text {* Most constants are already declared by HOL. *}
    16 
    16 
    17 consts
    17 consts
    18   assoc         :: "['a::times, 'a] => bool"              (infixl 50)
    18   assoc         :: "['a::times, 'a] => bool"              (infixl "assoc" 50)
    19   irred         :: "'a::{zero, one, times} => bool"
    19   irred         :: "'a::{zero, one, times} => bool"
    20   prime         :: "'a::{zero, one, times} => bool"
    20   prime         :: "'a::{zero, one, times} => bool"
    21 
    21 
    22 section {* Axioms *}
    22 section {* Axioms *}
    23 
    23