src/HOLCF/HOLCF.thy
author huffman
Sat, 02 Apr 2005 00:33:51 +0200
changeset 15651 4b393520846e
parent 15650 b37dc98fbbc5
child 15742 64eae3513064
permissions -rw-r--r--
Replaced continuity solver with new continuity simproc. Also removed cont lemmas from simp set, so that the simproc actually gets used.

(*  Title:      HOLCF/HOLCF.thy
    ID:         $Id$
    Author:     Franz Regensburger

Top theory for HOLCF system.
*)

theory HOLCF
imports Sprod Ssum Up Lift Discrete One Tr
begin

text {*
  Remove continuity lemmas from simp set, so continuity subgoals
  are handled by the @{text cont_proc} simplifier procedure.
*}
declare cont_lemmas1 [simp del]
declare cont_lemmas_ext [simp del]

end