src/LCF/ex/Ex3.thy
changeset 58977 9576b510f6a2
parent 58974 cbc2ac19d783
child 60770 240563fbf41d
equal deleted inserted replaced
58976:b38a54bbfbd6 58977:9576b510f6a2
     3 theory Ex3
     3 theory Ex3
     4 imports "../LCF"
     4 imports "../LCF"
     5 begin
     5 begin
     6 
     6 
     7 axiomatization
     7 axiomatization
     8   s     :: "'a => 'a" and
     8   s     :: "'a \<Rightarrow> 'a" and
     9   p     :: "'a => 'a => 'a"
     9   p     :: "'a \<Rightarrow> 'a \<Rightarrow> 'a"
    10 where
    10 where
    11   p_strict:     "p(UU) = UU" and
    11   p_strict:     "p(UU) = UU" and
    12   p_s:          "p(s(x),y) = s(p(x,y))"
    12   p_s:          "p(s(x),y) = s(p(x,y))"
    13 
    13 
    14 declare p_strict [simp] p_s [simp]
    14 declare p_strict [simp] p_s [simp]