src/HOL/ROOT
changeset 66946 3d8fd98c7c86
parent 66932 149025fecca0
child 66950 1a5e90026391
equal deleted inserted replaced
66945:b6f787a17fbe 66946:3d8fd98c7c86
    13 
    13 
    14 session "HOL-Proofs" (timing) = Pure +
    14 session "HOL-Proofs" (timing) = Pure +
    15   description {*
    15   description {*
    16     HOL-Main with explicit proof terms.
    16     HOL-Main with explicit proof terms.
    17   *}
    17   *}
    18   options [document = false, quick_and_dirty = false, record_proofs = 2, parallel_proofs = 0]
    18   options [quick_and_dirty = false, record_proofs = 2, parallel_proofs = 0]
    19   sessions
    19   sessions
    20     "HOL-Library"
    20     "HOL-Library"
    21   theories
    21   theories
    22     "HOL-Library.Old_Datatype"
    22     "HOL-Library.Old_Datatype"
    23 
    23 
   175 
   175 
   176     This is an extension of IMP with local variables and mutually recursive
   176     This is an extension of IMP with local variables and mutually recursive
   177     procedures. For documentation see "Hoare Logic for Mutual Recursion and
   177     procedures. For documentation see "Hoare Logic for Mutual Recursion and
   178     Local Variables" (http://isabelle.in.tum.de/Bali/papers/FSTTCS99.html).
   178     Local Variables" (http://isabelle.in.tum.de/Bali/papers/FSTTCS99.html).
   179   *}
   179   *}
   180   options [document = false]
       
   181   theories EvenOdd
   180   theories EvenOdd
   182 
   181 
   183 session "HOL-Data_Structures" (timing) in Data_Structures = HOL +
   182 session "HOL-Data_Structures" (timing) in Data_Structures = HOL +
   184   options [document_variants = document]
   183   options [document_variants = document]
   185   sessions
   184   sessions
   231   *}
   230   *}
   232   theories Hoare_Parallel
   231   theories Hoare_Parallel
   233   document_files "root.bib" "root.tex"
   232   document_files "root.bib" "root.tex"
   234 
   233 
   235 session "HOL-Codegenerator_Test" in Codegenerator_Test = "HOL-Number_Theory" +
   234 session "HOL-Codegenerator_Test" in Codegenerator_Test = "HOL-Number_Theory" +
   236   options [document = false, browser_info = false]
   235   options [browser_info = false]
   237   sessions
   236   sessions
   238     "HOL-Data_Structures"
   237     "HOL-Data_Structures"
   239     "HOL-ex"
   238     "HOL-ex"
   240   theories
   239   theories
   241     Generate
   240     Generate
   259     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
   258     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
   260     Author:     Jasmin Blanchette, TU Muenchen
   259     Author:     Jasmin Blanchette, TU Muenchen
   261 
   260 
   262     Testing Metis and Sledgehammer.
   261     Testing Metis and Sledgehammer.
   263   *}
   262   *}
   264   options [document = false]
       
   265   sessions
   263   sessions
   266     "HOL-Decision_Procs"
   264     "HOL-Decision_Procs"
   267   theories
   265   theories
   268     Abstraction
   266     Abstraction
   269     Big_O
   267     Big_O
   278 session "HOL-Nitpick_Examples" in Nitpick_Examples = "HOL-Library" +
   276 session "HOL-Nitpick_Examples" in Nitpick_Examples = "HOL-Library" +
   279   description {*
   277   description {*
   280     Author:     Jasmin Blanchette, TU Muenchen
   278     Author:     Jasmin Blanchette, TU Muenchen
   281     Copyright   2009
   279     Copyright   2009
   282   *}
   280   *}
   283   options [document = false]
       
   284   theories [quick_and_dirty] Nitpick_Examples
   281   theories [quick_and_dirty] Nitpick_Examples
   285 
   282 
   286 session "HOL-Algebra" (main timing) in Algebra = "HOL-Computational_Algebra" +
   283 session "HOL-Algebra" (main timing) in Algebra = "HOL-Computational_Algebra" +
   287   description {*
   284   description {*
   288     Author: Clemens Ballarin, started 24 September 1999
   285     Author: Clemens Ballarin, started 24 September 1999
   382 
   379 
   383 session "HOL-Decision_Procs" (timing) in Decision_Procs = "HOL-Algebra" +
   380 session "HOL-Decision_Procs" (timing) in Decision_Procs = "HOL-Algebra" +
   384   description {*
   381   description {*
   385     Various decision procedures, typically involving reflection.
   382     Various decision procedures, typically involving reflection.
   386   *}
   383   *}
   387   options [document = false]
       
   388   theories
   384   theories
   389     Decision_Procs
   385     Decision_Procs
   390 
   386 
   391 session "HOL-Proofs-ex" in "Proofs/ex" = "HOL-Proofs" +
   387 session "HOL-Proofs-ex" in "Proofs/ex" = "HOL-Proofs" +
   392   options [document = false]
       
   393   sessions
   388   sessions
   394     "HOL-Isar_Examples"
   389     "HOL-Isar_Examples"
   395   theories
   390   theories
   396     Hilbert_Classical
   391     Hilbert_Classical
   397     Proof_Terms
   392     Proof_Terms
   441 
   436 
   442     This is a simple exploratory implementation of Lambda-Prolog in HOL,
   437     This is a simple exploratory implementation of Lambda-Prolog in HOL,
   443     including some minimal examples (in Test.thy) and a more typical example of
   438     including some minimal examples (in Test.thy) and a more typical example of
   444     a little functional language and its type system.
   439     a little functional language and its type system.
   445   *}
   440   *}
   446   options [document = false]
       
   447   theories Test Type
   441   theories Test Type
   448 
   442 
   449 session "HOL-MicroJava" (timing) in MicroJava = "HOL-Library" +
   443 session "HOL-MicroJava" (timing) in MicroJava = "HOL-Library" +
   450   description {*
   444   description {*
   451     Formalization of a fragment of Java, together with a corresponding virtual
   445     Formalization of a fragment of Java, together with a corresponding virtual
   503     booktitle={Proc.\ TACAS Workshop},
   497     booktitle={Proc.\ TACAS Workshop},
   504     organization={Aarhus University, BRICS report},
   498     organization={Aarhus University, BRICS report},
   505     year=1995}
   499     year=1995}
   506     ftp://ftp.informatik.tu-muenchen.de/local/lehrstuhl/nipkow/tacas.dvi.gz
   500     ftp://ftp.informatik.tu-muenchen.de/local/lehrstuhl/nipkow/tacas.dvi.gz
   507   *}
   501   *}
   508   options [document = false]
       
   509   theories Solve
   502   theories Solve
   510 
   503 
   511 session "HOL-Lattice" in Lattice = HOL +
   504 session "HOL-Lattice" in Lattice = HOL +
   512   description {*
   505   description {*
   513     Author:     Markus Wenzel, TU Muenchen
   506     Author:     Markus Wenzel, TU Muenchen
   519 
   512 
   520 session "HOL-ex" (timing) in ex = "HOL-Number_Theory" +
   513 session "HOL-ex" (timing) in ex = "HOL-Number_Theory" +
   521   description {*
   514   description {*
   522     Miscellaneous examples for Higher-Order Logic.
   515     Miscellaneous examples for Higher-Order Logic.
   523   *}
   516   *}
   524   options [document = false]
       
   525   theories
   517   theories
   526     Adhoc_Overloading_Examples
   518     Adhoc_Overloading_Examples
   527     Antiquote
   519     Antiquote
   528     Argo_Examples
   520     Argo_Examples
   529     Arith_Examples
   521     Arith_Examples
   665 
   657 
   666 session "HOL-TLA" in TLA = HOL +
   658 session "HOL-TLA" in TLA = HOL +
   667   description {*
   659   description {*
   668     Lamport's Temporal Logic of Actions.
   660     Lamport's Temporal Logic of Actions.
   669   *}
   661   *}
   670   options [document = false]
       
   671   theories TLA
   662   theories TLA
   672 
   663 
   673 session "HOL-TLA-Inc" in "TLA/Inc" = "HOL-TLA" +
   664 session "HOL-TLA-Inc" in "TLA/Inc" = "HOL-TLA" +
   674   options [document = false]
       
   675   theories Inc
   665   theories Inc
   676 
   666 
   677 session "HOL-TLA-Buffer" in "TLA/Buffer" = "HOL-TLA" +
   667 session "HOL-TLA-Buffer" in "TLA/Buffer" = "HOL-TLA" +
   678   options [document = false]
       
   679   theories DBuffer
   668   theories DBuffer
   680 
   669 
   681 session "HOL-TLA-Memory" in "TLA/Memory" = "HOL-TLA" +
   670 session "HOL-TLA-Memory" in "TLA/Memory" = "HOL-TLA" +
   682   options [document = false]
       
   683   theories MemoryImplementation
   671   theories MemoryImplementation
   684 
   672 
   685 session "HOL-TPTP" in TPTP = "HOL-Library" +
   673 session "HOL-TPTP" in TPTP = "HOL-Library" +
   686   description {*
   674   description {*
   687     Author:     Jasmin Blanchette, TU Muenchen
   675     Author:     Jasmin Blanchette, TU Muenchen
   688     Author:     Nik Sultana, University of Cambridge
   676     Author:     Nik Sultana, University of Cambridge
   689     Copyright   2011
   677     Copyright   2011
   690 
   678 
   691     TPTP-related extensions.
   679     TPTP-related extensions.
   692   *}
   680   *}
   693   options [document = false]
       
   694   theories
   681   theories
   695     ATP_Theory_Export
   682     ATP_Theory_Export
   696     MaSh_Eval
   683     MaSh_Eval
   697     TPTP_Interpret
   684     TPTP_Interpret
   698     THF_Arith
   685     THF_Arith
   710     Dining_Cryptographers
   697     Dining_Cryptographers
   711     Koepf_Duermuth_Countermeasure
   698     Koepf_Duermuth_Countermeasure
   712     Measure_Not_CCC
   699     Measure_Not_CCC
   713 
   700 
   714 session "HOL-Nominal" in Nominal = "HOL-Library" +
   701 session "HOL-Nominal" in Nominal = "HOL-Library" +
   715   options [document = false]
       
   716   theories
   702   theories
   717     Nominal
   703     Nominal
   718 
   704 
   719 session "HOL-Nominal-Examples" (timing) in "Nominal/Examples" = "HOL-Nominal" +
   705 session "HOL-Nominal-Examples" (timing) in "Nominal/Examples" = "HOL-Nominal" +
   720   options [document = false]
       
   721   theories
   706   theories
   722     Class3
   707     Class3
   723     CK_Machine
   708     CK_Machine
   724     Compile
   709     Compile
   725     Contexts
   710     Contexts
   756 
   741 
   757 session "HOL-Datatype_Examples" (timing) in Datatype_Examples = "HOL-Library" +
   742 session "HOL-Datatype_Examples" (timing) in Datatype_Examples = "HOL-Library" +
   758   description {*
   743   description {*
   759     (Co)datatype Examples.
   744     (Co)datatype Examples.
   760   *}
   745   *}
   761   options [document = false]
       
   762   theories
   746   theories
   763     Compat
   747     Compat
   764     Lambda_Term
   748     Lambda_Term
   765     Process
   749     Process
   766     TreeFsetI
   750     TreeFsetI
   777 
   761 
   778 session "HOL-Corec_Examples" (timing) in Corec_Examples = "HOL-Library" +
   762 session "HOL-Corec_Examples" (timing) in Corec_Examples = "HOL-Library" +
   779   description {*
   763   description {*
   780     Corecursion Examples.
   764     Corecursion Examples.
   781   *}
   765   *}
   782   options [document = false]
       
   783   theories
   766   theories
   784     LFilter
   767     LFilter
   785     Paper_Examples
   768     Paper_Examples
   786     Stream_Processor
   769     Stream_Processor
   787     "Tests/Simple_Nesting"
   770     "Tests/Simple_Nesting"
   805     WordBitwise
   788     WordBitwise
   806     Bit_Comparison
   789     Bit_Comparison
   807   document_files "root.bib" "root.tex"
   790   document_files "root.bib" "root.tex"
   808 
   791 
   809 session "HOL-Word-Examples" in "Word/Examples" = "HOL-Word" +
   792 session "HOL-Word-Examples" in "Word/Examples" = "HOL-Word" +
   810   options [document = false]
       
   811   theories WordExamples
   793   theories WordExamples
   812 
   794 
   813 session "HOL-Statespace" in Statespace = HOL +
   795 session "HOL-Statespace" in Statespace = HOL +
   814   theories [skip_proofs = false]
   796   theories [skip_proofs = false]
   815     StateSpaceEx
   797     StateSpaceEx
   822   theories
   804   theories
   823     Nonstandard_Analysis
   805     Nonstandard_Analysis
   824   document_files "root.tex"
   806   document_files "root.tex"
   825 
   807 
   826 session "HOL-Nonstandard_Analysis-Examples" (timing) in "Nonstandard_Analysis/Examples" = "HOL-Nonstandard_Analysis" +
   808 session "HOL-Nonstandard_Analysis-Examples" (timing) in "Nonstandard_Analysis/Examples" = "HOL-Nonstandard_Analysis" +
   827   options [document = false]
       
   828   theories
   809   theories
   829     NSPrimes
   810     NSPrimes
   830 
   811 
   831 session "HOL-Mirabelle" in Mirabelle = HOL +
   812 session "HOL-Mirabelle" in Mirabelle = HOL +
   832   options [document = false]
       
   833   theories Mirabelle_Test
   813   theories Mirabelle_Test
   834 
   814 
   835 session "HOL-Mirabelle-ex" in "Mirabelle/ex" = "HOL-Mirabelle" +
   815 session "HOL-Mirabelle-ex" in "Mirabelle/ex" = "HOL-Mirabelle" +
   836   options [document = false, timeout = 60]
   816   options [timeout = 60]
   837   theories Ex
   817   theories Ex
   838 
   818 
   839 session "HOL-Word-SMT_Examples" (timing) in SMT_Examples = "HOL-Word" +
   819 session "HOL-Word-SMT_Examples" (timing) in SMT_Examples = "HOL-Word" +
   840   options [document = false, quick_and_dirty]
   820   options [quick_and_dirty]
   841   theories
   821   theories
   842     Boogie
   822     Boogie
   843     SMT_Examples
   823     SMT_Examples
   844     SMT_Word_Examples
   824     SMT_Word_Examples
   845     SMT_Tests
   825     SMT_Tests
   846 
   826 
   847 session "HOL-SPARK" (main) in "SPARK" = "HOL-Word" +
   827 session "HOL-SPARK" (main) in "SPARK" = "HOL-Word" +
   848   options [document = false]
       
   849   theories
   828   theories
   850     SPARK (global)
   829     SPARK (global)
   851 
   830 
   852 session "HOL-SPARK-Examples" in "SPARK/Examples" = "HOL-SPARK" +
   831 session "HOL-SPARK-Examples" in "SPARK/Examples" = "HOL-SPARK" +
   853   options [document = false, spark_prv = false]
   832   options [spark_prv = false]
   854   theories
   833   theories
   855     "Gcd/Greatest_Common_Divisor"
   834     "Gcd/Greatest_Common_Divisor"
   856     "Liseq/Longest_Increasing_Subsequence"
   835     "Liseq/Longest_Increasing_Subsequence"
   857     "RIPEMD-160/F"
   836     "RIPEMD-160/F"
   858     "RIPEMD-160/Hash"
   837     "RIPEMD-160/Hash"
   887     "root.tex"
   866     "root.tex"
   888     "Simple_Gcd.adb"
   867     "Simple_Gcd.adb"
   889     "Simple_Gcd.ads"
   868     "Simple_Gcd.ads"
   890 
   869 
   891 session "HOL-Mutabelle" in Mutabelle = "HOL-Library" +
   870 session "HOL-Mutabelle" in Mutabelle = "HOL-Library" +
   892   options [document = false]
       
   893   theories MutabelleExtra
   871   theories MutabelleExtra
   894 
   872 
   895 session "HOL-Quickcheck_Examples" (timing) in Quickcheck_Examples = "HOL-Library" +
   873 session "HOL-Quickcheck_Examples" (timing) in Quickcheck_Examples = "HOL-Library" +
   896   options [document = false]
       
   897   theories
   874   theories
   898     Quickcheck_Examples
   875     Quickcheck_Examples
   899     Quickcheck_Lattice_Examples
   876     Quickcheck_Lattice_Examples
   900     Completeness
   877     Completeness
   901     Quickcheck_Interfaces
   878     Quickcheck_Interfaces
   906 
   883 
   907 session "HOL-Quotient_Examples" (timing) in Quotient_Examples = "HOL-Algebra" +
   884 session "HOL-Quotient_Examples" (timing) in Quotient_Examples = "HOL-Algebra" +
   908   description {*
   885   description {*
   909     Author:     Cezary Kaliszyk and Christian Urban
   886     Author:     Cezary Kaliszyk and Christian Urban
   910   *}
   887   *}
   911   options [document = false]
       
   912   theories
   888   theories
   913     DList
   889     DList
   914     Quotient_FSet
   890     Quotient_FSet
   915     Quotient_Int
   891     Quotient_Int
   916     Quotient_Message
   892     Quotient_Message
   921     Lift_DList
   897     Lift_DList
   922     Int_Pow
   898     Int_Pow
   923     Lifting_Code_Dt_Test
   899     Lifting_Code_Dt_Test
   924 
   900 
   925 session "HOL-Predicate_Compile_Examples" (timing) in Predicate_Compile_Examples = "HOL-Library" +
   901 session "HOL-Predicate_Compile_Examples" (timing) in Predicate_Compile_Examples = "HOL-Library" +
   926   options [document = false]
       
   927   theories
   902   theories
   928     Examples
   903     Examples
   929     Predicate_Compile_Tests
   904     Predicate_Compile_Tests
   930     Predicate_Compile_Quickcheck_Examples
   905     Predicate_Compile_Quickcheck_Examples
   931     Specialisation_Examples
   906     Specialisation_Examples
   946 
   921 
   947 session "HOL-Types_To_Sets" in Types_To_Sets = HOL +
   922 session "HOL-Types_To_Sets" in Types_To_Sets = HOL +
   948   description {*
   923   description {*
   949     Experimental extension of Higher-Order Logic to allow translation of types to sets.
   924     Experimental extension of Higher-Order Logic to allow translation of types to sets.
   950   *}
   925   *}
   951   options [document = false]
       
   952   theories
   926   theories
   953     Types_To_Sets
   927     Types_To_Sets
   954     "Examples/Prerequisites"
   928     "Examples/Prerequisites"
   955     "Examples/Finite"
   929     "Examples/Finite"
   956     "Examples/T2_Spaces"
   930     "Examples/T2_Spaces"
   972     Fixrec_ex
   946     Fixrec_ex
   973     New_Domain
   947     New_Domain
   974   document_files "root.tex"
   948   document_files "root.tex"
   975 
   949 
   976 session "HOLCF-Library" in "HOLCF/Library" = HOLCF +
   950 session "HOLCF-Library" in "HOLCF/Library" = HOLCF +
   977   options [document = false]
       
   978   theories
   951   theories
   979     HOLCF_Library
   952     HOLCF_Library
   980     HOL_Cpo
   953     HOL_Cpo
   981 
   954 
   982 session "HOLCF-IMP" in "HOLCF/IMP" = HOLCF +
   955 session "HOLCF-IMP" in "HOLCF/IMP" = HOLCF +
   983   description {*
   956   description {*
   984     IMP -- A WHILE-language and its Semantics.
   957     IMP -- A WHILE-language and its Semantics.
   985 
   958 
   986     This is the HOLCF-based denotational semantics of a simple WHILE-language.
   959     This is the HOLCF-based denotational semantics of a simple WHILE-language.
   987   *}
   960   *}
   988   options [document = false]
       
   989   sessions
   961   sessions
   990     "HOL-IMP"
   962     "HOL-IMP"
   991   theories
   963   theories
   992     HoareEx
   964     HoareEx
   993   document_files "root.tex"
   965   document_files "root.tex"
   994 
   966 
   995 session "HOLCF-ex" in "HOLCF/ex" = "HOLCF-Library" +
   967 session "HOLCF-ex" in "HOLCF/ex" = "HOLCF-Library" +
   996   description {*
   968   description {*
   997     Miscellaneous examples for HOLCF.
   969     Miscellaneous examples for HOLCF.
   998   *}
   970   *}
   999   options [document = false]
       
  1000   theories
   971   theories
  1001     Dnat
   972     Dnat
  1002     Dagstuhl
   973     Dagstuhl
  1003     Focus_ex
   974     Focus_ex
  1004     Fix2
   975     Fix2
  1023     http://www4.in.tum.de/publ/html.php?e=15
   994     http://www4.in.tum.de/publ/html.php?e=15
  1024 
   995 
  1025     "Specification and Development of Interactive Systems: Focus on Streams,
   996     "Specification and Development of Interactive Systems: Focus on Streams,
  1026     Interfaces, and Refinement" http://www4.in.tum.de/publ/html.php?e=321
   997     Interfaces, and Refinement" http://www4.in.tum.de/publ/html.php?e=321
  1027   *}
   998   *}
  1028   options [document = false]
       
  1029   theories
   999   theories
  1030     Fstreams
  1000     Fstreams
  1031     FOCUS
  1001     FOCUS
  1032     Buffer_adm
  1002     Buffer_adm
  1033 
  1003 
  1040 
  1010 
  1041     The distribution contains simulation relations, temporal logic, and an
  1011     The distribution contains simulation relations, temporal logic, and an
  1042     abstraction theory. Everything is based upon a domain-theoretic model of
  1012     abstraction theory. Everything is based upon a domain-theoretic model of
  1043     finite and infinite sequences.
  1013     finite and infinite sequences.
  1044   *}
  1014   *}
  1045   options [document = false]
       
  1046   theories Abstraction
  1015   theories Abstraction
  1047 
  1016 
  1048 session "IOA-ABP" in "HOLCF/IOA/ABP" = IOA +
  1017 session "IOA-ABP" in "HOLCF/IOA/ABP" = IOA +
  1049   description {*
  1018   description {*
  1050     Author:     Olaf Mueller
  1019     Author:     Olaf Mueller
  1051 
  1020 
  1052     The Alternating Bit Protocol performed in I/O-Automata.
  1021     The Alternating Bit Protocol performed in I/O-Automata.
  1053   *}
  1022   *}
  1054   options [document = false]
       
  1055   theories
  1023   theories
  1056     Correctness
  1024     Correctness
  1057     Spec
  1025     Spec
  1058 
  1026 
  1059 session "IOA-NTP" in "HOLCF/IOA/NTP" = IOA +
  1027 session "IOA-NTP" in "HOLCF/IOA/NTP" = IOA +
  1061     Author:     Tobias Nipkow & Konrad Slind
  1029     Author:     Tobias Nipkow & Konrad Slind
  1062 
  1030 
  1063     A network transmission protocol, performed in the
  1031     A network transmission protocol, performed in the
  1064     I/O automata formalization by Olaf Mueller.
  1032     I/O automata formalization by Olaf Mueller.
  1065   *}
  1033   *}
  1066   options [document = false]
       
  1067   theories Correctness
  1034   theories Correctness
  1068 
  1035 
  1069 session "IOA-Storage" in "HOLCF/IOA/Storage" = IOA +
  1036 session "IOA-Storage" in "HOLCF/IOA/Storage" = IOA +
  1070   description {*
  1037   description {*
  1071     Author:     Olaf Mueller
  1038     Author:     Olaf Mueller
  1072 
  1039 
  1073     Memory storage case study.
  1040     Memory storage case study.
  1074   *}
  1041   *}
  1075   options [document = false]
       
  1076   theories Correctness
  1042   theories Correctness
  1077 
  1043 
  1078 session "IOA-ex" in "HOLCF/IOA/ex" = IOA +
  1044 session "IOA-ex" in "HOLCF/IOA/ex" = IOA +
  1079   description {*
  1045   description {*
  1080     Author:     Olaf Mueller
  1046     Author:     Olaf Mueller
  1081   *}
  1047   *}
  1082   options [document = false]
       
  1083   theories
  1048   theories
  1084     TrivEx
  1049     TrivEx
  1085     TrivEx2
  1050     TrivEx2