src/HOLCF/IOA/Modelcheck/MuIOAOracle.thy
author paulson
Wed, 19 Jul 2006 11:55:26 +0200
changeset 20153 6ff5d35749b0
parent 17244 0b2ff9541727
child 22819 a7b425bb668c
permissions -rw-r--r--
Fixed the bugs introduced by the last commit! Output is now *identical* to that produced by the old version, based on a-lists.


(* $Id$ *)

theory MuIOAOracle
imports MuIOA
begin

oracle sim_oracle ("term * thm list") =
  mk_sim_oracle

end