equal
deleted
inserted
replaced
180 where |
180 where |
181 "y \<noteq> A \<Longrightarrow> z \<noteq> B \<Longrightarrow> notAB (y, z)" |
181 "y \<noteq> A \<Longrightarrow> z \<noteq> B \<Longrightarrow> notAB (y, z)" |
182 |
182 |
183 values 5 "{y. notAB y}" |
183 values 5 "{y. notAB y}" |
184 |
184 |
|
185 section {* Example prolog conform variable names *} |
|
186 |
|
187 inductive equals :: "abc => abc => bool" |
|
188 where |
|
189 "equals y' y'" |
|
190 ML {* set Code_Prolog.trace *} |
|
191 values 1 "{(y, z). equals y z}" |
|
192 |
185 end |
193 end |