src/HOL/ROOT
changeset 63888 5a9a1985e9fb
parent 63885 a6cd18af8bf9
child 63920 003622e08379
equal deleted inserted replaced
63887:2d9c12eba726 63888:5a9a1985e9fb
    12     "Tools/Quickcheck/PNF_Narrowing_Engine.hs"
    12     "Tools/Quickcheck/PNF_Narrowing_Engine.hs"
    13   document_files
    13   document_files
    14     "root.bib"
    14     "root.bib"
    15     "root.tex"
    15     "root.tex"
    16 
    16 
    17 session "HOL-Proofs" = Pure +
    17 session "HOL-Proofs" (timing) = Pure +
    18   description {*
    18   description {*
    19     HOL-Main with explicit proof terms.
    19     HOL-Main with explicit proof terms.
    20   *}
    20   *}
    21   options [document = false, quick_and_dirty = false]
    21   options [document = false, quick_and_dirty = false]
    22   theories Proofs (*sequential change of global flag!*)
    22   theories Proofs (*sequential change of global flag!*)
    24   theories [checkpoint] "~~/src/HOL/Library/Old_Datatype"
    24   theories [checkpoint] "~~/src/HOL/Library/Old_Datatype"
    25   files
    25   files
    26     "Tools/Quickcheck/Narrowing_Engine.hs"
    26     "Tools/Quickcheck/Narrowing_Engine.hs"
    27     "Tools/Quickcheck/PNF_Narrowing_Engine.hs"
    27     "Tools/Quickcheck/PNF_Narrowing_Engine.hs"
    28 
    28 
    29 session "HOL-Library" (main) in Library = HOL +
    29 session "HOL-Library" (main timing) in Library = HOL +
    30   description {*
    30   description {*
    31     Classical Higher-order Logic -- batteries included.
    31     Classical Higher-order Logic -- batteries included.
    32   *}
    32   *}
    33   theories
    33   theories
    34     Library
    34     Library
   117     Comb
   117     Comb
   118     PropLog
   118     PropLog
   119     Com
   119     Com
   120   document_files "root.tex"
   120   document_files "root.tex"
   121 
   121 
   122 session "HOL-IMP" in IMP = HOL +
   122 session "HOL-IMP" (timing) in IMP = HOL +
   123   options [document_variants = document]
   123   options [document_variants = document]
   124   theories [document = false]
   124   theories [document = false]
   125     "~~/src/HOL/Library/While_Combinator"
   125     "~~/src/HOL/Library/While_Combinator"
   126     "~~/src/HOL/Library/Char_ord"
   126     "~~/src/HOL/Library/Char_ord"
   127     "~~/src/HOL/Library/List_lexord"
   127     "~~/src/HOL/Library/List_lexord"
   174     Local Variables" (http://isabelle.in.tum.de/Bali/papers/FSTTCS99.html).
   174     Local Variables" (http://isabelle.in.tum.de/Bali/papers/FSTTCS99.html).
   175   *}
   175   *}
   176   options [document = false]
   176   options [document = false]
   177   theories EvenOdd
   177   theories EvenOdd
   178 
   178 
   179 session "HOL-Data_Structures" in Data_Structures = HOL +
   179 session "HOL-Data_Structures" (timing) in Data_Structures = HOL +
   180   options [document_variants = document]
   180   options [document_variants = document]
   181   theories [document = false]
   181   theories [document = false]
   182     "Less_False"
   182     "Less_False"
   183     "~~/src/HOL/Library/Multiset"
   183     "~~/src/HOL/Library/Multiset"
   184     "~~/src/HOL/Library/Float"
   184     "~~/src/HOL/Library/Float"
   197 
   197 
   198 session "HOL-Import" in Import = HOL +
   198 session "HOL-Import" in Import = HOL +
   199   theories HOL_Light_Maps
   199   theories HOL_Light_Maps
   200   theories [condition = HOL_LIGHT_BUNDLE] HOL_Light_Import
   200   theories [condition = HOL_LIGHT_BUNDLE] HOL_Light_Import
   201 
   201 
   202 session "HOL-Number_Theory" in Number_Theory = HOL +
   202 session "HOL-Number_Theory" (timing) in Number_Theory = HOL +
   203   description {*
   203   description {*
   204     Fundamental Theorem of Arithmetic, Chinese Remainder Theorem, Fermat/Euler
   204     Fundamental Theorem of Arithmetic, Chinese Remainder Theorem, Fermat/Euler
   205     Theorem, Wilson's Theorem, some lemmas for Quadratic Reciprocity.
   205     Theorem, Wilson's Theorem, some lemmas for Quadratic Reciprocity.
   206   *}
   206   *}
   207   theories [document = false]
   207   theories [document = false]
   245     automatically from pre/post conditions and loop invariants).
   245     automatically from pre/post conditions and loop invariants).
   246   *}
   246   *}
   247   theories Hoare
   247   theories Hoare
   248   document_files "root.bib" "root.tex"
   248   document_files "root.bib" "root.tex"
   249 
   249 
   250 session "HOL-Hoare_Parallel" in Hoare_Parallel = HOL +
   250 session "HOL-Hoare_Parallel" (timing) in Hoare_Parallel = HOL +
   251   description {*
   251   description {*
   252     Verification of shared-variable imperative programs a la Owicki-Gries.
   252     Verification of shared-variable imperative programs a la Owicki-Gries.
   253     (verification conditions are generated automatically).
   253     (verification conditions are generated automatically).
   254   *}
   254   *}
   255   theories Hoare_Parallel
   255   theories Hoare_Parallel
   274   theories [condition = "ISABELLE_SCALA"]
   274   theories [condition = "ISABELLE_SCALA"]
   275     Code_Test_Scala
   275     Code_Test_Scala
   276   theories [condition = "ISABELLE_SMLNJ"]
   276   theories [condition = "ISABELLE_SMLNJ"]
   277     Code_Test_SMLNJ
   277     Code_Test_SMLNJ
   278 
   278 
   279 session "HOL-Metis_Examples" in Metis_Examples = HOL +
   279 session "HOL-Metis_Examples" (timing) in Metis_Examples = HOL +
   280   description {*
   280   description {*
   281     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
   281     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
   282     Author:     Jasmin Blanchette, TU Muenchen
   282     Author:     Jasmin Blanchette, TU Muenchen
   283 
   283 
   284     Testing Metis and Sledgehammer.
   284     Testing Metis and Sledgehammer.
   301     Copyright   2009
   301     Copyright   2009
   302   *}
   302   *}
   303   options [document = false]
   303   options [document = false]
   304   theories [quick_and_dirty] Nitpick_Examples
   304   theories [quick_and_dirty] Nitpick_Examples
   305 
   305 
   306 session "HOL-Algebra" (main) in Algebra = HOL +
   306 session "HOL-Algebra" (main timing) in Algebra = HOL +
   307   description {*
   307   description {*
   308     Author: Clemens Ballarin, started 24 September 1999
   308     Author: Clemens Ballarin, started 24 September 1999
   309 
   309 
   310     The Isabelle Algebraic Library.
   310     The Isabelle Algebraic Library.
   311   *}
   311   *}
   325     Divisibility         (* Rings *)
   325     Divisibility         (* Rings *)
   326     IntRing              (* Ideals and residue classes *)
   326     IntRing              (* Ideals and residue classes *)
   327     UnivPoly             (* Polynomials *)
   327     UnivPoly             (* Polynomials *)
   328   document_files "root.bib" "root.tex"
   328   document_files "root.bib" "root.tex"
   329 
   329 
   330 session "HOL-Auth" in Auth = HOL +
   330 session "HOL-Auth" (timing) in Auth = HOL +
   331   description {*
   331   description {*
   332     A new approach to verifying authentication protocols.
   332     A new approach to verifying authentication protocols.
   333   *}
   333   *}
   334   theories
   334   theories
   335     Auth_Shared
   335     Auth_Shared
   337     "Smartcard/Auth_Smartcard"
   337     "Smartcard/Auth_Smartcard"
   338     "Guard/Auth_Guard_Shared"
   338     "Guard/Auth_Guard_Shared"
   339     "Guard/Auth_Guard_Public"
   339     "Guard/Auth_Guard_Public"
   340   document_files "root.tex"
   340   document_files "root.tex"
   341 
   341 
   342 session "HOL-UNITY" in UNITY = "HOL-Auth" +
   342 session "HOL-UNITY" (timing) in UNITY = "HOL-Auth" +
   343   description {*
   343   description {*
   344     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
   344     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
   345     Copyright   1998  University of Cambridge
   345     Copyright   1998  University of Cambridge
   346 
   346 
   347     Verifying security protocols using Chandy and Misra's UNITY formalism.
   347     Verifying security protocols using Chandy and Misra's UNITY formalism.
   399     "~~/src/HOL/Library/Monad_Syntax"
   399     "~~/src/HOL/Library/Monad_Syntax"
   400     "~~/src/HOL/Library/LaTeXsugar"
   400     "~~/src/HOL/Library/LaTeXsugar"
   401   theories Imperative_HOL_ex
   401   theories Imperative_HOL_ex
   402   document_files "root.bib" "root.tex"
   402   document_files "root.bib" "root.tex"
   403 
   403 
   404 session "HOL-Decision_Procs" in Decision_Procs = HOL +
   404 session "HOL-Decision_Procs" (timing) in Decision_Procs = HOL +
   405   description {*
   405   description {*
   406     Various decision procedures, typically involving reflection.
   406     Various decision procedures, typically involving reflection.
   407   *}
   407   *}
   408   options [document = false]
   408   options [document = false]
   409   theories Decision_Procs
   409   theories Decision_Procs
   413   theories
   413   theories
   414     Hilbert_Classical
   414     Hilbert_Classical
   415     Proof_Terms
   415     Proof_Terms
   416     XML_Data
   416     XML_Data
   417 
   417 
   418 session "HOL-Proofs-Extraction" in "Proofs/Extraction" = "HOL-Proofs" +
   418 session "HOL-Proofs-Extraction" (timing) in "Proofs/Extraction" = "HOL-Proofs" +
   419   description {*
   419   description {*
   420     Examples for program extraction in Higher-Order Logic.
   420     Examples for program extraction in Higher-Order Logic.
   421   *}
   421   *}
   422   options [parallel_proofs = 0, quick_and_dirty = false]
   422   options [parallel_proofs = 0, quick_and_dirty = false]
   423   theories [document = false]
   423   theories [document = false]
   431     Higman_Extraction
   431     Higman_Extraction
   432     Pigeonhole
   432     Pigeonhole
   433     Euclid
   433     Euclid
   434   document_files "root.bib" "root.tex"
   434   document_files "root.bib" "root.tex"
   435 
   435 
   436 session "HOL-Proofs-Lambda" in "Proofs/Lambda" = "HOL-Proofs" +
   436 session "HOL-Proofs-Lambda" (timing) in "Proofs/Lambda" = "HOL-Proofs" +
   437   description {*
   437   description {*
   438     Lambda Calculus in de Bruijn's Notation.
   438     Lambda Calculus in de Bruijn's Notation.
   439 
   439 
   440     This session defines lambda-calculus terms with de Bruijn indixes and
   440     This session defines lambda-calculus terms with de Bruijn indixes and
   441     proves confluence of beta, eta and beta+eta.
   441     proves confluence of beta, eta and beta+eta.
   465     a little functional language and its type system.
   465     a little functional language and its type system.
   466   *}
   466   *}
   467   options [document = false]
   467   options [document = false]
   468   theories Test Type
   468   theories Test Type
   469 
   469 
   470 session "HOL-MicroJava" in MicroJava = HOL +
   470 session "HOL-MicroJava" (timing) in MicroJava = HOL +
   471   description {*
   471   description {*
   472     Formalization of a fragment of Java, together with a corresponding virtual
   472     Formalization of a fragment of Java, together with a corresponding virtual
   473     machine and a specification of its bytecode verifier and a lightweight
   473     machine and a specification of its bytecode verifier and a lightweight
   474     bytecode verifier, including proofs of type-safety.
   474     bytecode verifier, including proofs of type-safety.
   475   *}
   475   *}
   487     Hoare Logic for a tiny fragment of Java.
   487     Hoare Logic for a tiny fragment of Java.
   488   *}
   488   *}
   489   theories Example
   489   theories Example
   490   document_files "root.bib" "root.tex"
   490   document_files "root.bib" "root.tex"
   491 
   491 
   492 session "HOL-Bali" in Bali = HOL +
   492 session "HOL-Bali" (timing) in Bali = HOL +
   493   theories
   493   theories
   494     AxExample
   494     AxExample
   495     AxSound
   495     AxSound
   496     AxCompl
   496     AxCompl
   497     Trans
   497     Trans
   669     Eisbach
   669     Eisbach
   670     Tests
   670     Tests
   671     Examples
   671     Examples
   672     Examples_FOL
   672     Examples_FOL
   673 
   673 
   674 session "HOL-SET_Protocol" in SET_Protocol = HOL +
   674 session "HOL-SET_Protocol" (timing) in SET_Protocol = HOL +
   675   description {*
   675   description {*
   676     Verification of the SET Protocol.
   676     Verification of the SET Protocol.
   677   *}
   677   *}
   678   theories [document = false] "~~/src/HOL/Library/Nat_Bijection"
   678   theories [document = false] "~~/src/HOL/Library/Nat_Bijection"
   679   theories SET_Protocol
   679   theories SET_Protocol
   721     THF_Arith
   721     THF_Arith
   722     TPTP_Proof_Reconstruction
   722     TPTP_Proof_Reconstruction
   723   theories
   723   theories
   724     ATP_Problem_Import
   724     ATP_Problem_Import
   725 
   725 
   726 session "HOL-Analysis" (main) in Analysis = HOL +
   726 session "HOL-Analysis" (main timing) in Analysis = HOL +
   727   theories
   727   theories
   728     Analysis
   728     Analysis
   729   document_files
   729   document_files
   730     "root.tex"
   730     "root.tex"
   731 
   731 
   732 session "HOL-Analysis-ex" in "Analysis/ex" = "HOL-Analysis" +
   732 session "HOL-Analysis-ex" in "Analysis/ex" = "HOL-Analysis" +
   733   theories
   733   theories
   734     Approximations
   734     Approximations
   735 
   735 
   736 session "HOL-Probability" in "Probability" = "HOL-Analysis" +
   736 session "HOL-Probability" (timing) in "Probability" = "HOL-Analysis" +
   737   theories [document = false]
   737   theories [document = false]
   738     "~~/src/HOL/Library/Countable"
   738     "~~/src/HOL/Library/Countable"
   739     "~~/src/HOL/Library/Permutation"
   739     "~~/src/HOL/Library/Permutation"
   740     "~~/src/HOL/Library/Order_Continuity"
   740     "~~/src/HOL/Library/Order_Continuity"
   741     "~~/src/HOL/Library/Diagonal_Subsequence"
   741     "~~/src/HOL/Library/Diagonal_Subsequence"
   742     "~~/src/HOL/Library/Finite_Map"
   742     "~~/src/HOL/Library/Finite_Map"
   743   theories
   743   theories
   744     Probability
   744     Probability
   745   document_files "root.tex"
   745   document_files "root.tex"
   746 
   746 
   747 session "HOL-Probability-ex" in "Probability/ex" = "HOL-Probability" +
   747 session "HOL-Probability-ex" (timing) in "Probability/ex" = "HOL-Probability" +
   748   theories
   748   theories
   749     "Dining_Cryptographers"
   749     "Dining_Cryptographers"
   750     "Koepf_Duermuth_Countermeasure"
   750     "Koepf_Duermuth_Countermeasure"
   751     "Measure_Not_CCC"
   751     "Measure_Not_CCC"
   752 
   752 
   753 session "HOL-Nominal" in Nominal = HOL +
   753 session "HOL-Nominal" in Nominal = HOL +
   754   options [document = false]
   754   options [document = false]
   755   theories Nominal
   755   theories Nominal
   756 
   756 
   757 session "HOL-Nominal-Examples" in "Nominal/Examples" = "HOL-Nominal" +
   757 session "HOL-Nominal-Examples" (timing) in "Nominal/Examples" = "HOL-Nominal" +
   758   options [document = false]
   758   options [document = false]
   759   theories
   759   theories
   760     Class3
   760     Class3
   761     CK_Machine
   761     CK_Machine
   762     Compile
   762     Compile
   778     Weakening
   778     Weakening
   779     W
   779     W
   780   theories [quick_and_dirty]
   780   theories [quick_and_dirty]
   781     VC_Condition
   781     VC_Condition
   782 
   782 
   783 session "HOL-Cardinals" in Cardinals = HOL +
   783 session "HOL-Cardinals" (timing) in Cardinals = HOL +
   784   description {*
   784   description {*
   785     Ordinals and Cardinals, Full Theories.
   785     Ordinals and Cardinals, Full Theories.
   786   *}
   786   *}
   787   options [document = false]
   787   options [document = false]
   788   theories
   788   theories
   791   document_files
   791   document_files
   792     "intro.tex"
   792     "intro.tex"
   793     "root.tex"
   793     "root.tex"
   794     "root.bib"
   794     "root.bib"
   795 
   795 
   796 session "HOL-Datatype_Examples" in Datatype_Examples = HOL +
   796 session "HOL-Datatype_Examples" (timing) in Datatype_Examples = HOL +
   797   description {*
   797   description {*
   798     (Co)datatype Examples.
   798     (Co)datatype Examples.
   799   *}
   799   *}
   800   options [document = false]
   800   options [document = false]
   801   theories
   801   theories
   812     Misc_Codatatype
   812     Misc_Codatatype
   813     Misc_Datatype
   813     Misc_Datatype
   814     Misc_Primcorec
   814     Misc_Primcorec
   815     Misc_Primrec
   815     Misc_Primrec
   816 
   816 
   817 session "HOL-Corec_Examples" in Corec_Examples = HOL +
   817 session "HOL-Corec_Examples" (timing) in Corec_Examples = HOL +
   818   description {*
   818   description {*
   819     Corecursion Examples.
   819     Corecursion Examples.
   820   *}
   820   *}
   821   options [document = false]
   821   options [document = false]
   822   theories
   822   theories
   833     "Tests/Small_Concrete"
   833     "Tests/Small_Concrete"
   834     "Tests/Stream_Friends"
   834     "Tests/Stream_Friends"
   835     "Tests/TLList_Friends"
   835     "Tests/TLList_Friends"
   836     "Tests/Type_Class"
   836     "Tests/Type_Class"
   837 
   837 
   838 session "HOL-Word" (main) in Word = HOL +
   838 session "HOL-Word" (main timing) in Word = HOL +
   839   theories Word
   839   theories Word
   840   document_files "root.bib" "root.tex"
   840   document_files "root.bib" "root.tex"
   841 
   841 
   842 session "HOL-Word-Examples" in "Word/Examples" = "HOL-Word" +
   842 session "HOL-Word-Examples" in "Word/Examples" = "HOL-Word" +
   843   options [document = false]
   843   options [document = false]
   846 session "HOL-Statespace" in Statespace = HOL +
   846 session "HOL-Statespace" in Statespace = HOL +
   847   theories [skip_proofs = false]
   847   theories [skip_proofs = false]
   848     StateSpaceEx
   848     StateSpaceEx
   849   document_files "root.tex"
   849   document_files "root.tex"
   850 
   850 
   851 session "HOL-Nonstandard_Analysis" in Nonstandard_Analysis = HOL +
   851 session "HOL-Nonstandard_Analysis" (timing) in Nonstandard_Analysis = HOL +
   852   description {*
   852   description {*
   853     Nonstandard analysis.
   853     Nonstandard analysis.
   854   *}
   854   *}
   855   theories
   855   theories
   856     Nonstandard_Analysis
   856     Nonstandard_Analysis
   857   document_files "root.tex"
   857   document_files "root.tex"
   858 
   858 
   859 session "HOL-Nonstandard_Analysis-Examples" in "Nonstandard_Analysis/Examples" = "HOL-Nonstandard_Analysis" +
   859 session "HOL-Nonstandard_Analysis-Examples" (timing) in "Nonstandard_Analysis/Examples" = "HOL-Nonstandard_Analysis" +
   860   options [document = false]
   860   options [document = false]
   861   theories NSPrimes
   861   theories NSPrimes
   862 
   862 
   863 session "HOL-Mirabelle" in Mirabelle = HOL +
   863 session "HOL-Mirabelle" in Mirabelle = HOL +
   864   options [document = false]
   864   options [document = false]
   866 
   866 
   867 session "HOL-Mirabelle-ex" in "Mirabelle/ex" = "HOL-Mirabelle" +
   867 session "HOL-Mirabelle-ex" in "Mirabelle/ex" = "HOL-Mirabelle" +
   868   options [document = false, timeout = 60]
   868   options [document = false, timeout = 60]
   869   theories Ex
   869   theories Ex
   870 
   870 
   871 session "HOL-Word-SMT_Examples" in SMT_Examples = "HOL-Word" +
   871 session "HOL-Word-SMT_Examples" (timing) in SMT_Examples = "HOL-Word" +
   872   options [document = false, quick_and_dirty]
   872   options [document = false, quick_and_dirty]
   873   theories
   873   theories
   874     Boogie
   874     Boogie
   875     SMT_Examples
   875     SMT_Examples
   876     SMT_Word_Examples
   876     SMT_Word_Examples
   975 
   975 
   976 session "HOL-Mutabelle" in Mutabelle = HOL +
   976 session "HOL-Mutabelle" in Mutabelle = HOL +
   977   options [document = false]
   977   options [document = false]
   978   theories MutabelleExtra
   978   theories MutabelleExtra
   979 
   979 
   980 session "HOL-Quickcheck_Examples" in Quickcheck_Examples = HOL +
   980 session "HOL-Quickcheck_Examples" (timing) in Quickcheck_Examples = HOL +
   981   options [document = false]
   981   options [document = false]
   982   theories
   982   theories
   983     Quickcheck_Examples
   983     Quickcheck_Examples
   984     Quickcheck_Lattice_Examples
   984     Quickcheck_Lattice_Examples
   985     Completeness
   985     Completeness
   987     Quickcheck_Nesting_Example
   987     Quickcheck_Nesting_Example
   988   theories [condition = ISABELLE_GHC]
   988   theories [condition = ISABELLE_GHC]
   989     Hotel_Example
   989     Hotel_Example
   990     Quickcheck_Narrowing_Examples
   990     Quickcheck_Narrowing_Examples
   991 
   991 
   992 session "HOL-Quotient_Examples" in Quotient_Examples = HOL +
   992 session "HOL-Quotient_Examples" (timing) in Quotient_Examples = HOL +
   993   description {*
   993   description {*
   994     Author:     Cezary Kaliszyk and Christian Urban
   994     Author:     Cezary Kaliszyk and Christian Urban
   995   *}
   995   *}
   996   options [document = false]
   996   options [document = false]
   997   theories
   997   theories
  1005     Quotient_Rat
  1005     Quotient_Rat
  1006     Lift_DList
  1006     Lift_DList
  1007     Int_Pow
  1007     Int_Pow
  1008     Lifting_Code_Dt_Test
  1008     Lifting_Code_Dt_Test
  1009 
  1009 
  1010 session "HOL-Predicate_Compile_Examples" in Predicate_Compile_Examples = HOL +
  1010 session "HOL-Predicate_Compile_Examples" (timing) in Predicate_Compile_Examples = HOL +
  1011   options [document = false]
  1011   options [document = false]
  1012   theories
  1012   theories
  1013     Examples
  1013     Examples
  1014     Predicate_Compile_Tests
  1014     Predicate_Compile_Tests
  1015     Predicate_Compile_Quickcheck_Examples
  1015     Predicate_Compile_Quickcheck_Examples
  1027     Lambda_Example
  1027     Lambda_Example
  1028     List_Examples
  1028     List_Examples
  1029   theories [condition = ISABELLE_SWIPL, quick_and_dirty]
  1029   theories [condition = ISABELLE_SWIPL, quick_and_dirty]
  1030     Reg_Exp_Example
  1030     Reg_Exp_Example
  1031 
  1031 
  1032 session HOLCF (main) in HOLCF = HOL +
  1032 session HOLCF (main timing) in HOLCF = HOL +
  1033   description {*
  1033   description {*
  1034     Author:     Franz Regensburger
  1034     Author:     Franz Regensburger
  1035     Author:     Brian Huffman
  1035     Author:     Brian Huffman
  1036 
  1036 
  1037     HOLCF -- a semantic extension of HOL by the LCF logic.
  1037     HOLCF -- a semantic extension of HOL by the LCF logic.
  1103   theories
  1103   theories
  1104     Fstreams
  1104     Fstreams
  1105     FOCUS
  1105     FOCUS
  1106     Buffer_adm
  1106     Buffer_adm
  1107 
  1107 
  1108 session IOA in "HOLCF/IOA" = HOLCF +
  1108 session IOA (timing) in "HOLCF/IOA" = HOLCF +
  1109   description {*
  1109   description {*
  1110     Author:     Olaf Mueller
  1110     Author:     Olaf Mueller
  1111     Copyright   1997 TU München
  1111     Copyright   1997 TU München
  1112 
  1112 
  1113     A formalization of I/O automata in HOLCF.
  1113     A formalization of I/O automata in HOLCF.