src/HOLCF/HOLCF.thy
author huffman
Fri, 10 Apr 2009 17:39:53 -0700
changeset 30911 7809cbaa1b61
parent 30910 a7cc0ef93269
child 31076 99fe356cbbc2
permissions -rw-r--r--
domain package: simplify internal proofs of con_rews
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
1479
21eb5e156d91 expanded tabs
clasohm
parents: 1274
diff changeset
     1
(*  Title:      HOLCF/HOLCF.thy
21eb5e156d91 expanded tabs
clasohm
parents: 1274
diff changeset
     2
    Author:     Franz Regensburger
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
     3
16841
228d663cc9b3 use all files in HOLCF.thy;
wenzelm
parents: 16054
diff changeset
     4
HOLCF -- a semantic extension of HOL by the LCF logic.
243
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
     5
*)
c22b85994e17 Franz Regensburger's Higher-Order Logic of Computable Functions embedding LCF
nipkow
parents:
diff changeset
     6
15650
b37dc98fbbc5 converted to new-style theory
huffman
parents: 15576
diff changeset
     7
theory HOLCF
29130
685c9e05a6ab new theory Dsum: cpo of disjoint sum
huffman
parents: 28892
diff changeset
     8
imports
29534
247e4c816004 rename Dsum.thy to Sum_Cpo.thy
huffman
parents: 29530
diff changeset
     9
  Domain ConvexPD Algebraic Universal Sum_Cpo Main
16841
228d663cc9b3 use all files in HOLCF.thy;
wenzelm
parents: 16054
diff changeset
    10
uses
228d663cc9b3 use all files in HOLCF.thy;
wenzelm
parents: 16054
diff changeset
    11
  "holcf_logic.ML"
23152
9497234a2743 moved HOLCF tools to canonical place;
wenzelm
parents: 19105
diff changeset
    12
  "Tools/adm_tac.ML"
15650
b37dc98fbbc5 converted to new-style theory
huffman
parents: 15576
diff changeset
    13
begin
b37dc98fbbc5 converted to new-style theory
huffman
parents: 15576
diff changeset
    14
25904
8161f137b0e9 new theory of powerdomains
huffman
parents: 23152
diff changeset
    15
defaultsort pcpo
8161f137b0e9 new theory of powerdomains
huffman
parents: 23152
diff changeset
    16
26339
7825c83c9eff eliminated change_claset/simpset;
wenzelm
parents: 25904
diff changeset
    17
declaration {* fn _ =>
7825c83c9eff eliminated change_claset/simpset;
wenzelm
parents: 25904
diff changeset
    18
  Simplifier.map_ss (fn simpset => simpset addSolver
17612
5b37787d2d9e adm_tac/cont_tacRs: proper simpset;
wenzelm
parents: 16841
diff changeset
    19
    (mk_solver' "adm_tac" (fn ss =>
30603
71180005f251 proper context for prove_cont/adm_tac;
wenzelm
parents: 29542
diff changeset
    20
      Adm.adm_tac (Simplifier.the_context ss)
71180005f251 proper context for prove_cont/adm_tac;
wenzelm
parents: 29542
diff changeset
    21
        (cut_facts_tac (Simplifier.prems_of_ss ss) THEN' cont_tacRs ss))));
16841
228d663cc9b3 use all files in HOLCF.thy;
wenzelm
parents: 16054
diff changeset
    22
*}
228d663cc9b3 use all files in HOLCF.thy;
wenzelm
parents: 16054
diff changeset
    23
15650
b37dc98fbbc5 converted to new-style theory
huffman
parents: 15576
diff changeset
    24
end