src/HOLCF/IOA/Modelcheck/MuIOAOracle.thy
author aspinall
Fri, 30 Sep 2005 18:18:34 +0200
changeset 17740 fc385ce6187d
parent 17244 0b2ff9541727
child 22819 a7b425bb668c
permissions -rw-r--r--
Add icon for interface.


(* $Id$ *)

theory MuIOAOracle
imports MuIOA
begin

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

end