equal
deleted
inserted
replaced
289 |
289 |
290 code_pred big_step . |
290 code_pred big_step . |
291 |
291 |
292 thm big_step.equation |
292 thm big_step.equation |
293 |
293 |
|
294 definition list :: "(nat \<Rightarrow> 'a) \<Rightarrow> nat \<Rightarrow> 'a list" where |
|
295 "list s n = map s [0 ..< n]" |
|
296 |
|
297 values [expected "{[42, (43 :: nat)]}"] "{list s 2|s. (SKIP, nth [42, 43]) \<Rightarrow> s}" |
|
298 |
|
299 |
294 subsection {* CCS *} |
300 subsection {* CCS *} |
295 |
301 |
296 text{* This example formalizes finite CCS processes without communication or |
302 text{* This example formalizes finite CCS processes without communication or |
297 recursion. For simplicity, labels are natural numbers. *} |
303 recursion. For simplicity, labels are natural numbers. *} |
298 |
304 |