3 session HOL (main) = Pure +
5 Classical Higher-order Logic.
11 "Tools/Quickcheck/Narrowing_Engine.hs"
12 "Tools/Quickcheck/PNF_Narrowing_Engine.hs"
17 session "HOL-Proofs" (slow) = Pure +
19 HOL-Main with explicit proof terms.
21 options [document = false, quick_and_dirty = false]
22 theories Proofs (*sequential change of global flag!*)
23 theories "~~/src/HOL/Library/Old_Datatype"
25 "Tools/Quickcheck/Narrowing_Engine.hs"
26 "Tools/Quickcheck/PNF_Narrowing_Engine.hs"
28 session "HOL-Library" (main) in Library = HOL +
30 Classical Higher-order Logic -- batteries included.
35 (*conflicting type class instantiations*)
41 (*data refinements and dependent applications*)
46 Code_Real_Approx_By_Float
57 document_files "root.bib" "root.tex"
59 session "HOL-Hahn_Banach" in Hahn_Banach = HOL +
61 Author: Gertrud Bauer, TU Munich
63 The Hahn-Banach theorem for real vector spaces.
65 This is the proof of the Hahn-Banach theorem for real vectorspaces,
66 following H. Heuser, Funktionalanalysis, p. 228 -232. The Hahn-Banach
67 theorem is one of the fundamental theorems of functional analysis. It is a
68 conclusion of Zorn's lemma.
70 Two different formaulations of the theorem are presented, one for general
71 real vectorspaces and its application to normed vectorspaces.
73 The theorem says, that every continous linearform, defined on arbitrary
74 subspaces (not only one-dimensional subspaces), can be extended to a
75 continous linearform on the whole vectorspace.
78 document_files "root.bib" "root.tex"
80 session "HOL-Induct" in Induct = HOL +
82 Examples of (Co)Inductive Definitions.
84 Comb proves the Church-Rosser theorem for combinators (see
85 http://www.cl.cam.ac.uk/ftp/papers/reports/TR396-lcp-generic-automatic-proof-tools.ps.gz).
87 Mutil is the famous Mutilated Chess Board problem (see
88 http://www.cl.cam.ac.uk/ftp/papers/reports/TR394-lcp-mutilated-chess-board.dvi.gz).
90 PropLog proves the completeness of a formalization of propositional logic
92 http://www.cl.cam.ac.uk/Research/Reports/TR312-lcp-set-II.ps.gz).
94 Exp demonstrates the use of iterated inductive definitions to reason about
95 mutually recursive relations.
97 theories [document = false]
98 "~~/src/HOL/Library/Old_Datatype"
99 theories [quick_and_dirty]
113 document_files "root.tex"
115 session "HOL-IMP" in IMP = HOL +
116 options [document_variants = document]
117 theories [document = false]
118 "~~/src/Tools/Permanent_Interpretation"
119 "~~/src/HOL/Library/While_Combinator"
120 "~~/src/HOL/Library/Char_ord"
121 "~~/src/HOL/Library/List_lexord"
122 "~~/src/HOL/Library/Quotient_List"
123 "~~/src/HOL/Library/Extended"
147 "Abs_Int_ITP/Abs_Int1_parity_ITP"
148 "Abs_Int_ITP/Abs_Int1_const_ITP"
149 "Abs_Int_ITP/Abs_Int3_ITP"
150 "Abs_Int_Den/Abs_Int_den2"
156 document_files "root.bib" "root.tex"
158 session "HOL-IMPP" in IMPP = HOL +
160 Author: David von Oheimb
163 IMPP -- An imperative language with procedures.
165 This is an extension of IMP with local variables and mutually recursive
166 procedures. For documentation see "Hoare Logic for Mutual Recursion and
167 Local Variables" (http://isabelle.in.tum.de/Bali/papers/FSTTCS99.html).
169 options [document = false]
172 session "HOL-Data_Structures" in Data_Structures = HOL +
173 options [document_variants = document]
174 theories [document = false]
183 document_files "root.tex" "root.bib"
185 session "HOL-Import" in Import = HOL +
186 theories HOL_Light_Maps
187 theories [condition = HOL_LIGHT_BUNDLE] HOL_Light_Import
189 session "HOL-Number_Theory" in Number_Theory = HOL +
191 Fundamental Theorem of Arithmetic, Chinese Remainder Theorem, Fermat/Euler
192 Theorem, Wilson's Theorem, some lemmas for Quadratic Reciprocity.
194 theories [document = false]
195 "~~/src/HOL/Library/FuncSet"
196 "~~/src/HOL/Library/Multiset"
197 "~~/src/HOL/Algebra/Ring"
198 "~~/src/HOL/Algebra/FiniteProduct"
208 session "HOL-Old_Number_Theory" in Old_Number_Theory = HOL +
210 Fundamental Theorem of Arithmetic, Chinese Remainder Theorem, Fermat/Euler
211 Theorem, Wilson's Theorem, Quadratic Reciprocity.
213 theories [document = false]
214 "~~/src/HOL/Library/Infinite_Set"
215 "~~/src/HOL/Library/Permutation"
222 Quadratic_Reciprocity
229 session "HOL-Hoare" in Hoare = HOL +
231 Verification of imperative programs (verification conditions are generated
232 automatically from pre/post conditions and loop invariants).
235 document_files "root.bib" "root.tex"
237 session "HOL-Hoare_Parallel" in Hoare_Parallel = HOL +
239 Verification of shared-variable imperative programs a la Owicki-Gries.
240 (verification conditions are generated automatically).
242 theories Hoare_Parallel
243 document_files "root.bib" "root.tex"
245 session "HOL-Codegenerator_Test" in Codegenerator_Test = "HOL-Library" +
246 options [condition = ML_SYSTEM_POLYML, document = false, browser_info = false]
251 Generate_Efficient_Datastructures
253 theories [condition = ISABELLE_GHC]
255 theories [condition = ISABELLE_MLTON]
257 theories [condition = ISABELLE_OCAMLC]
259 theories [condition = ISABELLE_POLYML]
261 theories [condition = ISABELLE_SCALA]
263 theories [condition = ISABELLE_SMLNJ]
266 session "HOL-Metis_Examples" in Metis_Examples = HOL +
268 Author: Lawrence C Paulson, Cambridge University Computer Laboratory
269 Author: Jasmin Blanchette, TU Muenchen
271 Testing Metis and Sledgehammer.
273 options [document = false]
285 session "HOL-Nitpick_Examples" in Nitpick_Examples = HOL +
287 Author: Jasmin Blanchette, TU Muenchen
290 options [document = false]
291 theories [quick_and_dirty] Nitpick_Examples
293 session "HOL-Algebra" (main) in Algebra = HOL +
295 Author: Clemens Ballarin, started 24 September 1999
297 The Isabelle Algebraic Library.
299 theories [document = false]
300 (* Preliminaries from set and number theory *)
301 "~~/src/HOL/Library/FuncSet"
302 "~~/src/HOL/Number_Theory/Primes"
303 "~~/src/HOL/Library/Permutation"
305 (*** New development, based on explicit structures ***)
307 FiniteProduct (* Product operator for commutative groups *)
308 Sylow (* Sylow's theorem *)
309 Bij (* Automorphism Groups *)
312 Divisibility (* Rings *)
313 IntRing (* Ideals and residue classes *)
314 UnivPoly (* Polynomials *)
315 document_files "root.bib" "root.tex"
317 session "HOL-Auth" in Auth = HOL +
319 A new approach to verifying authentication protocols.
324 "Smartcard/Auth_Smartcard"
325 "Guard/Auth_Guard_Shared"
326 "Guard/Auth_Guard_Public"
327 document_files "root.tex"
329 session "HOL-UNITY" in UNITY = "HOL-Auth" +
331 Author: Lawrence C Paulson, Cambridge University Computer Laboratory
332 Copyright 1998 University of Cambridge
334 Verifying security protocols using Chandy and Misra's UNITY formalism.
337 (*Basic meta-theory*)
340 (*Simple examples: no composition*)
349 "Simple/Reachability"
351 (*Verifying security protocols using UNITY*)
354 (*Example of composition*)
357 (*Universal properties examples*)
371 document_files "root.tex"
373 session "HOL-Unix" in Unix = HOL +
374 options [print_mode = "no_brackets,no_type_brackets"]
376 document_files "root.bib" "root.tex"
378 session "HOL-ZF" in ZF = HOL +
379 theories MainZF Games
380 document_files "root.tex"
382 session "HOL-Imperative_HOL" in Imperative_HOL = HOL +
383 options [print_mode = "iff,no_brackets"]
384 theories [document = false]
385 "~~/src/HOL/Library/Countable"
386 "~~/src/HOL/Library/Monad_Syntax"
387 "~~/src/HOL/Library/LaTeXsugar"
388 theories Imperative_HOL_ex
389 document_files "root.bib" "root.tex"
391 session "HOL-Decision_Procs" in Decision_Procs = HOL +
393 Various decision procedures, typically involving reflection.
395 options [condition = ML_SYSTEM_POLYML, document = false]
396 theories Decision_Procs
398 session "HOL-Proofs-ex" in "Proofs/ex" = "HOL-Proofs" +
399 options [document = false, parallel_proofs = 0]
404 session "HOL-Proofs-Extraction" in "Proofs/Extraction" = "HOL-Proofs" +
406 Examples for program extraction in Higher-Order Logic.
408 options [condition = ML_SYSTEM_POLYML, parallel_proofs = 0, quick_and_dirty = false]
409 theories [document = false]
410 "~~/src/HOL/Library/Code_Target_Numeral"
411 "~~/src/HOL/Library/Monad_Syntax"
412 "~~/src/HOL/Number_Theory/Primes"
413 "~~/src/HOL/Number_Theory/UniqueFactorization"
414 "~~/src/HOL/Library/State_Monad"
416 Greatest_Common_Divisor
421 document_files "root.bib" "root.tex"
423 session "HOL-Proofs-Lambda" in "Proofs/Lambda" = "HOL-Proofs" +
425 Lambda Calculus in de Bruijn's Notation.
427 This session defines lambda-calculus terms with de Bruijn indixes and
428 proves confluence of beta, eta and beta+eta.
430 The paper "More Church-Rosser Proofs (in Isabelle/HOL)" describes the whole
431 theory (see http://www.in.tum.de/~nipkow/pubs/jar2001.html).
433 options [print_mode = "no_brackets", parallel_proofs = 0, quick_and_dirty = false]
434 theories [document = false]
435 "~~/src/HOL/Library/Code_Target_Int"
441 document_files "root.bib" "root.tex"
443 session "HOL-Prolog" in Prolog = HOL +
445 Author: David von Oheimb (based on a lecture on Lambda Prolog by Nadathur)
447 A bare-bones implementation of Lambda-Prolog.
449 This is a simple exploratory implementation of Lambda-Prolog in HOL,
450 including some minimal examples (in Test.thy) and a more typical example of
451 a little functional language and its type system.
453 options [document = false]
456 session "HOL-MicroJava" in MicroJava = HOL +
458 Formalization of a fragment of Java, together with a corresponding virtual
459 machine and a specification of its bytecode verifier and a lightweight
460 bytecode verifier, including proofs of type-safety.
462 theories [document = false]
463 "~~/src/HOL/Library/While_Combinator"
471 session "HOL-NanoJava" in NanoJava = HOL +
473 Hoare Logic for a tiny fragment of Java.
476 document_files "root.bib" "root.tex"
478 session "HOL-Bali" in Bali = HOL +
485 document_files "root.tex"
487 session "HOL-IOA" in IOA = HOL +
489 Author: Tobias Nipkow and Konrad Slind and Olaf Müller
490 Copyright 1994--1996 TU Muenchen
492 The meta-theory of I/O-Automata in HOL. This formalization has been
493 significantly changed and extended, see HOLCF/IOA. There are also the
494 proofs of two communication protocols which formerly have been here.
496 @inproceedings{Nipkow-Slind-IOA,
497 author={Tobias Nipkow and Konrad Slind},
498 title={{I/O} Automata in {Isabelle/HOL}},
499 booktitle={Proc.\ TYPES Workshop 1994},
503 ftp://ftp.informatik.tu-muenchen.de/local/lehrstuhl/nipkow/ioa.ps.gz
507 @inproceedings{Mueller-Nipkow,
508 author={Olaf M\"uller and Tobias Nipkow},
509 title={Combining Model Checking and Deduction for {I/O}-Automata},
510 booktitle={Proc.\ TACAS Workshop},
511 organization={Aarhus University, BRICS report},
513 ftp://ftp.informatik.tu-muenchen.de/local/lehrstuhl/nipkow/tacas.dvi.gz
515 options [document = false]
518 session "HOL-Lattice" in Lattice = HOL +
520 Author: Markus Wenzel, TU Muenchen
522 Basic theory of lattices and orders.
524 theories CompleteLattice
525 document_files "root.tex"
527 session "HOL-ex" in ex = HOL +
529 Miscellaneous examples for Higher-Order Logic.
531 options [condition = ML_SYSTEM_POLYML]
532 theories [document = false]
533 "~~/src/HOL/Library/State_Monad"
534 Code_Binary_Nat_examples
535 "~~/src/HOL/Library/FuncSet"
537 Normalization_by_Evaluation
541 "~~/src/HOL/Library/FinFun_Syntax"
542 "~~/src/HOL/Library/Refute"
543 "~~/src/HOL/Library/Transitive_Closure_Table"
547 Adhoc_Overloading_Examples
557 While_Combinator_Example
591 Transitive_Closure_Table_Ex
599 List_to_Set_Comprehension_Examples
604 Set_Comprehension_Pointfree_Examples
607 Simps_Case_Conv_Examples
616 theories [skip_proofs = false]
618 theories [condition = ISABELLE_FULL_TEST]
620 document_files "root.bib" "root.tex"
622 session "HOL-Isar_Examples" in Isar_Examples = HOL +
624 Miscellaneous Isabelle/Isar examples for Higher-Order Logic.
626 theories [document = false]
627 "~~/src/HOL/Library/Lattice_Syntax"
628 "../Number_Theory/Primes"
640 Mutilated_Checkerboard
645 theories [quick_and_dirty]
646 Structured_Statements
652 session "HOL-Eisbach" in Eisbach = HOL +
654 The Eisbach proof method language and "match" method.
661 session "HOL-SET_Protocol" in SET_Protocol = HOL +
663 Verification of the SET Protocol.
665 theories [document = false] "~~/src/HOL/Library/Nat_Bijection"
666 theories SET_Protocol
667 document_files "root.tex"
669 session "HOL-Matrix_LP" in Matrix_LP = HOL +
671 Two-dimensional matrices and linear programming.
674 document_files "root.tex"
676 session "HOL-TLA" in TLA = HOL +
678 Lamport's Temporal Logic of Actions.
680 options [document = false]
683 session "HOL-TLA-Inc" in "TLA/Inc" = "HOL-TLA" +
684 options [document = false]
687 session "HOL-TLA-Buffer" in "TLA/Buffer" = "HOL-TLA" +
688 options [document = false]
691 session "HOL-TLA-Memory" in "TLA/Memory" = "HOL-TLA" +
692 options [document = false]
693 theories MemoryImplementation
695 session "HOL-TPTP" in TPTP = HOL +
697 Author: Jasmin Blanchette, TU Muenchen
698 Author: Nik Sultana, University of Cambridge
701 TPTP-related extensions.
703 options [condition = ML_SYSTEM_POLYML, document = false]
709 TPTP_Proof_Reconstruction
713 session "HOL-Multivariate_Analysis" (main) in Multivariate_Analysis = HOL +
715 Multivariate_Analysis
718 Complex_Analysis_Basics
719 Complex_Transcendental
724 session "HOL-Multivariate_Analysis-ex" in "Multivariate_Analysis/ex" = "HOL-Multivariate_Analysis" +
728 session "HOL-Probability" in "Probability" = "HOL-Multivariate_Analysis" +
729 theories [document = false]
730 "~~/src/HOL/Library/Countable"
731 "~~/src/HOL/Library/Permutation"
732 "~~/src/HOL/Library/Order_Continuity"
733 "~~/src/HOL/Library/Diagonal_Subsequence"
736 "ex/Dining_Cryptographers"
737 "ex/Koepf_Duermuth_Countermeasure"
739 document_files "root.tex"
741 session "HOL-Nominal" in Nominal = HOL +
742 options [document = false]
745 session "HOL-Nominal-Examples" in "Nominal/Examples" = "HOL-Nominal" +
746 options [condition = ML_SYSTEM_POLYML, document = false]
768 theories [quick_and_dirty]
771 session "HOL-Cardinals" in Cardinals = HOL +
773 Ordinals and Cardinals, Full Theories.
775 options [document = false]
784 session "HOL-Datatype_Examples" in Datatype_Examples = HOL +
786 (Co)datatype Examples, including large ones from John Harrison.
788 options [document = false]
790 "~~/src/HOL/Library/Old_Datatype"
795 "Derivation_Trees/Gram_Lang"
796 "Derivation_Trees/Parallel"
804 theories [condition = ISABELLE_FULL_TEST]
809 session "HOL-Word" (main) in Word = HOL +
811 document_files "root.bib" "root.tex"
813 session "HOL-Word-Examples" in "Word/Examples" = "HOL-Word" +
814 options [document = false]
815 theories WordExamples
817 session "HOL-Statespace" in Statespace = HOL +
818 theories [skip_proofs = false]
820 document_files "root.tex"
822 session "HOL-NSA" in NSA = HOL +
824 Nonstandard analysis.
826 theories Hypercomplex
827 document_files "root.tex"
829 session "HOL-NSA-Examples" in "NSA/Examples" = "HOL-NSA" +
830 options [document = false]
833 session "HOL-Mirabelle" in Mirabelle = HOL +
834 options [document = false]
835 theories Mirabelle_Test
837 session "HOL-Mirabelle-ex" in "Mirabelle/ex" = "HOL-Mirabelle" +
838 options [condition = ML_SYSTEM_POLYML, document = false, timeout = 60]
841 session "HOL-Word-SMT_Examples" in SMT_Examples = "HOL-Word" +
842 options [document = false, quick_and_dirty]
847 theories [condition = ISABELLE_FULL_TEST]
850 "Boogie_Dijkstra.certs"
853 "SMT_Word_Examples.certs"
856 session "HOL-SPARK" (main) in "SPARK" = "HOL-Word" +
857 options [document = false]
860 session "HOL-SPARK-Examples" in "SPARK/Examples" = "HOL-SPARK" +
861 options [document = false, spark_prv = false]
863 "Gcd/Greatest_Common_Divisor"
865 "Liseq/Longest_Increasing_Subsequence"
879 "Gcd/greatest_common_divisor/g_c_d.fdl"
880 "Gcd/greatest_common_divisor/g_c_d.rls"
881 "Gcd/greatest_common_divisor/g_c_d.siv"
882 "Liseq/liseq/liseq_length.fdl"
883 "Liseq/liseq/liseq_length.rls"
884 "Liseq/liseq/liseq_length.siv"
885 "RIPEMD-160/rmd/f.fdl"
886 "RIPEMD-160/rmd/f.rls"
887 "RIPEMD-160/rmd/f.siv"
888 "RIPEMD-160/rmd/hash.fdl"
889 "RIPEMD-160/rmd/hash.rls"
890 "RIPEMD-160/rmd/hash.siv"
891 "RIPEMD-160/rmd/k_l.fdl"
892 "RIPEMD-160/rmd/k_l.rls"
893 "RIPEMD-160/rmd/k_l.siv"
894 "RIPEMD-160/rmd/k_r.fdl"
895 "RIPEMD-160/rmd/k_r.rls"
896 "RIPEMD-160/rmd/k_r.siv"
897 "RIPEMD-160/rmd/r_l.fdl"
898 "RIPEMD-160/rmd/r_l.rls"
899 "RIPEMD-160/rmd/r_l.siv"
900 "RIPEMD-160/rmd/round.fdl"
901 "RIPEMD-160/rmd/round.rls"
902 "RIPEMD-160/rmd/round.siv"
903 "RIPEMD-160/rmd/r_r.fdl"
904 "RIPEMD-160/rmd/r_r.rls"
905 "RIPEMD-160/rmd/r_r.siv"
906 "RIPEMD-160/rmd/s_l.fdl"
907 "RIPEMD-160/rmd/s_l.rls"
908 "RIPEMD-160/rmd/s_l.siv"
909 "RIPEMD-160/rmd/s_r.fdl"
910 "RIPEMD-160/rmd/s_r.rls"
911 "RIPEMD-160/rmd/s_r.siv"
913 session "HOL-SPARK-Manual" in "SPARK/Manual" = "HOL-SPARK" +
914 options [show_question_marks = false, spark_prv = false]
921 "complex_types_app/initialize.fdl"
922 "complex_types_app/initialize.rls"
923 "complex_types_app/initialize.siv"
924 "loop_invariant/proc1.fdl"
925 "loop_invariant/proc1.rls"
926 "loop_invariant/proc1.siv"
927 "loop_invariant/proc2.fdl"
928 "loop_invariant/proc2.rls"
929 "loop_invariant/proc2.siv"
930 "simple_greatest_common_divisor/g_c_d.fdl"
931 "simple_greatest_common_divisor/g_c_d.rls"
932 "simple_greatest_common_divisor/g_c_d.siv"
935 "complex_types_app.adb"
936 "complex_types_app.ads"
947 session "HOL-Mutabelle" in Mutabelle = HOL +
948 options [document = false]
949 theories MutabelleExtra
951 session "HOL-Quickcheck_Examples" in Quickcheck_Examples = HOL +
952 options [document = false]
955 Quickcheck_Lattice_Examples
957 Quickcheck_Interfaces
958 theories [condition = ISABELLE_GHC]
960 Quickcheck_Narrowing_Examples
962 session "HOL-Quickcheck_Benchmark" in Quickcheck_Benchmark = HOL +
963 theories [condition = ISABELLE_FULL_TEST, quick_and_dirty]
964 Find_Unused_Assms_Examples
965 Needham_Schroeder_No_Attacker_Example
966 Needham_Schroeder_Guided_Attacker_Example
967 Needham_Schroeder_Unguided_Attacker_Example
969 session "HOL-Quotient_Examples" in Quotient_Examples = HOL +
971 Author: Cezary Kaliszyk and Christian Urban
973 options [document = false]
987 session "HOL-Predicate_Compile_Examples" in Predicate_Compile_Examples = HOL +
988 options [document = false]
991 Predicate_Compile_Tests
992 Predicate_Compile_Quickcheck_Examples
993 Specialisation_Examples
996 (* FIXME since 21-Jul-2011
997 Hotel_Example_Small_Generator *)
1000 theories [condition = "ISABELLE_SWIPL"]
1001 Code_Prolog_Examples
1002 Context_Free_Grammar_Example
1003 Hotel_Example_Prolog
1006 theories [condition = "ISABELLE_SWIPL", quick_and_dirty]
1009 session HOLCF (main) in HOLCF = HOL +
1011 Author: Franz Regensburger
1012 Author: Brian Huffman
1014 HOLCF -- a semantic extension of HOL by the LCF logic.
1016 theories [document = false]
1017 "~~/src/HOL/Library/Nat_Bijection"
1018 "~~/src/HOL/Library/Countable"
1023 document_files "root.tex"
1025 session "HOLCF-Tutorial" in "HOLCF/Tutorial" = HOLCF +
1030 document_files "root.tex"
1032 session "HOLCF-Library" in "HOLCF/Library" = HOLCF +
1033 options [document = false]
1034 theories HOLCF_Library
1036 session "HOLCF-IMP" in "HOLCF/IMP" = HOLCF +
1038 IMP -- A WHILE-language and its Semantics.
1040 This is the HOLCF-based denotational semantics of a simple WHILE-language.
1042 options [document = false]
1044 document_files "root.tex"
1046 session "HOLCF-ex" in "HOLCF/ex" = HOLCF +
1048 Miscellaneous examples for HOLCF.
1050 options [document = false]
1064 session "HOLCF-FOCUS" in "HOLCF/FOCUS" = HOLCF +
1066 FOCUS: a theory of stream-processing functions Isabelle/HOLCF.
1068 For introductions to FOCUS, see
1070 "The Design of Distributed Systems - An Introduction to FOCUS"
1071 http://www4.in.tum.de/publ/html.php?e=2
1073 "Specification and Refinement of a Buffer of Length One"
1074 http://www4.in.tum.de/publ/html.php?e=15
1076 "Specification and Development of Interactive Systems: Focus on Streams,
1077 Interfaces, and Refinement" http://www4.in.tum.de/publ/html.php?e=321
1079 options [document = false]
1085 session IOA in "HOLCF/IOA" = HOLCF +
1087 Author: Olaf Mueller
1088 Copyright 1997 TU München
1090 A formalization of I/O automata in HOLCF.
1092 The distribution contains simulation relations, temporal logic, and an
1093 abstraction theory. Everything is based upon a domain-theoretic model of
1094 finite and infinite sequences.
1096 options [document = false]
1097 theories "meta_theory/Abstraction"
1099 session "IOA-ABP" in "HOLCF/IOA/ABP" = IOA +
1101 Author: Olaf Mueller
1103 The Alternating Bit Protocol performed in I/O-Automata.
1105 options [document = false]
1110 session "IOA-NTP" in "HOLCF/IOA/NTP" = IOA +
1112 Author: Tobias Nipkow & Konrad Slind
1114 A network transmission protocol, performed in the
1115 I/O automata formalization by Olaf Mueller.
1117 options [document = false]
1118 theories Correctness
1120 session "IOA-Storage" in "HOLCF/IOA/Storage" = IOA +
1122 Author: Olaf Mueller
1124 Memory storage case study.
1126 options [document = false]
1127 theories Correctness
1129 session "IOA-ex" in "HOLCF/IOA/ex" = IOA +
1131 Author: Olaf Mueller
1133 options [document = false]
1138 session "HOL-Record_Benchmark" in Record_Benchmark = HOL +
1140 Some benchmark on large record.
1142 options [document = false]
1143 theories [condition = ISABELLE_FULL_TEST]