equal
deleted
inserted
replaced
520 code_pred [random_dseq] filter2 . |
520 code_pred [random_dseq] filter2 . |
521 |
521 |
522 thm filter2.equation |
522 thm filter2.equation |
523 thm filter2.random_dseq_equation |
523 thm filter2.random_dseq_equation |
524 |
524 |
525 (* |
|
526 inductive filter3 |
525 inductive filter3 |
527 for P |
526 for P |
528 where |
527 where |
529 "List.filter P xs = ys ==> filter3 P xs ys" |
528 "List.filter P xs = ys ==> filter3 P xs ys" |
530 |
529 |
531 code_pred (expected_modes: (o => bool) => i => o => bool, (o => bool) => i => i => bool , (i => bool) => i => o => bool, (i => bool) => i => i => bool) [skip_proof] filter3 . |
530 code_pred (expected_modes: (o => bool) => i => o => bool, (o => bool) => i => i => bool , (i => bool) => i => o => bool, (i => bool) => i => i => bool) [skip_proof] filter3 . |
532 |
531 |
533 code_pred [dseq] filter3 . |
532 code_pred filter3 . |
534 thm filter3.dseq_equation |
533 thm filter3.equation |
535 *) |
534 |
536 (* |
535 (* |
537 inductive filter4 |
536 inductive filter4 |
538 where |
537 where |
539 "List.filter P xs = ys ==> filter4 P xs ys" |
538 "List.filter P xs = ys ==> filter4 P xs ys" |
540 |
539 |