src/FOL/ex/Prolog.thy
changeset 352 fd3ab8bcb69d
parent 0 a5a9c433f639
child 1322 9b3d3362a048
equal deleted inserted replaced
351:1718ce07a584 352:fd3ab8bcb69d
     7 
     7 
     8 Inherits from FOL the class term, the type o, and the coercion Trueprop
     8 Inherits from FOL the class term, the type o, and the coercion Trueprop
     9 *)
     9 *)
    10 
    10 
    11 Prolog = FOL +
    11 Prolog = FOL +
    12 types   list 1
    12 types   'a list
    13 arities list    :: (term)term
    13 arities list    :: (term)term
    14 consts  Nil     :: "'a list"
    14 consts  Nil     :: "'a list"
    15         ":"     :: "['a, 'a list]=> 'a list"            (infixr 60)
    15         ":"     :: "['a, 'a list]=> 'a list"            (infixr 60)
    16         app     :: "['a list, 'a list, 'a list] => o"
    16         app     :: "['a list, 'a list, 'a list] => o"
    17         rev     :: "['a list, 'a list] => o"
    17         rev     :: "['a list, 'a list] => o"