src/HOLCF/Library/HOLCF_Library.thy
author blanchet
Mon, 04 Oct 2010 09:05:15 +0200
changeset 39930 61aa00205a88
parent 39143 d80990d8b909
child 39999 e3948547b541
permissions -rw-r--r--
hack in MESON to make it less likely that variables (e.g. "x") get renamed (e.g. "xa") when resolving

theory HOLCF_Library
imports
  List_Cpo
  Stream
  Strict_Fun
  Sum_Cpo
begin

end