author | lcp |
Tue, 25 Apr 1995 11:14:03 +0200 | |
changeset 1072 | 0140ff702b23 |
parent 1050 | 0c36c6a52a1d |
child 1138 | 82fd99d5a6ff |
permissions | -rw-r--r-- |
(* Title: HOL/IOA/ABP/Correctness.thy ID: $Id$ Author: Tobias Nipkow & Olaf Mueller Copyright 1994 TU Muenchen The main correctness proof: System_fin implements System *) Correctness = Solve + Env + Impl + Impl_finite + consts reduce :: "'a list => 'a list" primrec reduce List.list reduce_Nil "reduce [] = []" reduce_Cons "reduce(x#xs) = \ \ (case xs of \ \ [] => [x] \ \ | y#ys => (if (x=y) \ \ then reduce xs \ \ else (x#(reduce xs))))" end