src/HOL/Prolog/Test.thy
changeset 41310 65631ca437c9
parent 36319 8feb2c4bef1a
child 42793 88bee9f6eec7
equal deleted inserted replaced
41309:2e9bf718a7a1 41310:65631ca437c9
    35 
    35 
    36   bob     :: person
    36   bob     :: person
    37   sue     :: person
    37   sue     :: person
    38   ned     :: person
    38   ned     :: person
    39 
    39 
    40   "23"    :: nat          ("23")
    40   nat23   :: nat          ("23")
    41   "24"    :: nat          ("24")
    41   nat24   :: nat          ("24")
    42   "25"    :: nat          ("25")
    42   nat25   :: nat          ("25")
    43 
    43 
    44   age     :: "[person, nat]                          => bool"
    44   age     :: "[person, nat]                          => bool"
    45 
    45 
    46   eq      :: "['a, 'a]                               => bool"
    46   eq      :: "['a, 'a]                               => bool"
    47 
    47