src/ZF/Univ.thy
changeset 796 357a1f2dd07e
parent 753 ec86863e87c8
child 1155 928a16e02f9f
equal deleted inserted replaced
795:d689e796d186 796:357a1f2dd07e
     9 
     9 
    10 NOTE: univ(A) could be a translation; would simplify many proofs!
    10 NOTE: univ(A) could be a translation; would simplify many proofs!
    11   But Ind_Syntax.univ refers to the constant "univ"
    11   But Ind_Syntax.univ refers to the constant "univ"
    12 *)
    12 *)
    13 
    13 
    14 Univ = Arith + Sum + "mono" +
    14 Univ = Arith + Sum + Finite + "mono" +
    15 consts
    15 consts
    16     Vfrom       :: "[i,i]=>i"
    16     Vfrom       :: "[i,i]=>i"
    17     Vset        :: "i=>i"
    17     Vset        :: "i=>i"
    18     Vrec        :: "[i, [i,i]=>i] =>i"
    18     Vrec        :: "[i, [i,i]=>i] =>i"
    19     univ        :: "i=>i"
    19     univ        :: "i=>i"