src/HOLCF/HOLCF.thy
author urbanc
Fri, 17 Nov 2006 17:32:30 +0100
changeset 21405 26b51f724fe6
parent 19105 3aabd46340e0
child 23152 9497234a2743
permissions -rw-r--r--
added an intro lemma for freshness of products; set up the simplifier so that it can deal with the compact and long notation for freshness constraints (FIXME: it should also be able to deal with the special case of freshness of atoms)

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

HOLCF -- a semantic extension of HOL by the LCF logic.
*)

theory HOLCF
imports Sprod Ssum Up Lift Discrete One Tr Domain Main
uses
  "holcf_logic.ML"
  "cont_consts.ML"
  "domain/library.ML"
  "domain/syntax.ML"
  "domain/axioms.ML"
  "domain/theorems.ML"
  "domain/extender.ML"
  "adm_tac.ML"

begin

ML_setup {*
  change_simpset (fn simpset => simpset addSolver
    (mk_solver' "adm_tac" (fn ss =>
      adm_tac (cut_facts_tac (Simplifier.prems_of_ss ss) THEN' cont_tacRs ss))));
*}

end