src/HOL/ROOT
changeset 48483 9bfb6978eb80
parent 48481 2c828c830ad7
child 48486 691d0b44a793
equal deleted inserted replaced
48482:45137257399a 48483:9bfb6978eb80
   112 session IMPP = HOL +
   112 session IMPP = HOL +
   113   description {*
   113   description {*
   114     Author:     David von Oheimb
   114     Author:     David von Oheimb
   115     Copyright   1999 TUM
   115     Copyright   1999 TUM
   116   *}
   116   *}
       
   117   options [document = false]
   117   theories EvenOdd
   118   theories EvenOdd
   118 
   119 
   119 session Import = HOL +
   120 session Import = HOL +
   120   options [document_graph]
   121   options [document_graph]
   121   theories HOL_Light_Maps
   122   theories HOL_Light_Maps
   122   theories [condition = HOL_LIGHT_BUNDLE] HOL_Light_Import
   123   theories [condition = HOL_LIGHT_BUNDLE] HOL_Light_Import
   123 
   124 
   124 session Number_Theory = HOL +
   125 session Number_Theory = HOL +
       
   126   options [document = false]
   125   theories Number_Theory
   127   theories Number_Theory
   126 
   128 
   127 session Old_Number_Theory = HOL +
   129 session Old_Number_Theory = HOL +
   128   options [document_graph]
   130   options [document_graph]
   129   theories [document = false]
   131   theories [document = false]
   158     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
   160     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
   159     Author:     Jasmin Blanchette, TU Muenchen
   161     Author:     Jasmin Blanchette, TU Muenchen
   160 
   162 
   161     Testing Metis and Sledgehammer.
   163     Testing Metis and Sledgehammer.
   162   *}
   164   *}
       
   165   options [document = false]
   163   theories
   166   theories
   164     Abstraction
   167     Abstraction
   165     Big_O
   168     Big_O
   166     Binary_Tree
   169     Binary_Tree
   167     Clausification
   170     Clausification
   174 session Nitpick_Examples = HOL +
   177 session Nitpick_Examples = HOL +
   175   description {*
   178   description {*
   176     Author:     Jasmin Blanchette, TU Muenchen
   179     Author:     Jasmin Blanchette, TU Muenchen
   177     Copyright   2009
   180     Copyright   2009
   178   *}
   181   *}
       
   182   options [document = false]
   179   theories [quick_and_dirty] Nitpick_Examples
   183   theories [quick_and_dirty] Nitpick_Examples
   180 
   184 
   181 session Algebra = HOL +
   185 session Algebra = HOL +
   182   description {*
   186   description {*
   183     Author: Clemens Ballarin, started 24 September 1999
   187     Author: Clemens Ballarin, started 24 September 1999
   284     "~~/src/HOL/Library/LaTeXsugar"
   288     "~~/src/HOL/Library/LaTeXsugar"
   285   theories Imperative_HOL_ex
   289   theories Imperative_HOL_ex
   286   files "document/root.bib" "document/root.tex"
   290   files "document/root.bib" "document/root.tex"
   287 
   291 
   288 session Decision_Procs = HOL +
   292 session Decision_Procs = HOL +
       
   293   options [document = false]
   289   theories Decision_Procs
   294   theories Decision_Procs
   290 
   295 
   291 session ex in "Proofs/ex" = "HOL-Proofs" +
   296 session ex in "Proofs/ex" = "HOL-Proofs" +
   292   options [proofs = 2, parallel_proofs = 0]
   297   options [document = false, proofs = 2, parallel_proofs = 0]
   293   theories Hilbert_Classical
   298   theories Hilbert_Classical
   294 
   299 
   295 session Extraction in "Proofs/Extraction" = "HOL-Proofs" +
   300 session Extraction in "Proofs/Extraction" = "HOL-Proofs" +
   296   description {* Examples for program extraction in Higher-Order Logic *}
   301   description {* Examples for program extraction in Higher-Order Logic *}
   297   options [proofs = 2, parallel_proofs = 0]
   302   options [proofs = 2, parallel_proofs = 0]
   322 
   327 
   323 session Prolog = HOL +
   328 session Prolog = HOL +
   324   description {*
   329   description {*
   325     Author:   David von Oheimb (based on a lecture on Lambda Prolog by Nadathur)
   330     Author:   David von Oheimb (based on a lecture on Lambda Prolog by Nadathur)
   326   *}
   331   *}
       
   332   options [document = false]
   327   theories Test Type
   333   theories Test Type
   328 
   334 
   329 session MicroJava = HOL +
   335 session MicroJava = HOL +
   330   options [document_graph]
   336   options [document_graph]
   331   theories [document = false] "~~/src/HOL/Library/While_Combinator"
   337   theories [document = false] "~~/src/HOL/Library/While_Combinator"
   373     booktitle={Proc.\ TACAS Workshop},
   379     booktitle={Proc.\ TACAS Workshop},
   374     organization={Aarhus University, BRICS report},
   380     organization={Aarhus University, BRICS report},
   375     year=1995}
   381     year=1995}
   376     ftp://ftp.informatik.tu-muenchen.de/local/lehrstuhl/nipkow/tacas.dvi.gz
   382     ftp://ftp.informatik.tu-muenchen.de/local/lehrstuhl/nipkow/tacas.dvi.gz
   377   *}
   383   *}
       
   384   options [document = false]
   378   theories Solve
   385   theories Solve
   379 
   386 
   380 session Lattice = HOL +
   387 session Lattice = HOL +
   381   description {*
   388   description {*
   382     Author:     Markus Wenzel, TU Muenchen
   389     Author:     Markus Wenzel, TU Muenchen
   507   theories Cplex
   514   theories Cplex
   508   files "document/root.tex"
   515   files "document/root.tex"
   509 
   516 
   510 session TLA! = HOL +
   517 session TLA! = HOL +
   511   description {* The Temporal Logic of Actions *}
   518   description {* The Temporal Logic of Actions *}
       
   519   options [document = false]
   512   theories TLA
   520   theories TLA
   513 
   521 
   514 session Inc in "TLA/Inc" = TLA +
   522 session Inc in "TLA/Inc" = TLA +
       
   523   options [document = false]
   515   theories Inc
   524   theories Inc
   516 
   525 
   517 session Buffer in "TLA/Buffer" = TLA +
   526 session Buffer in "TLA/Buffer" = TLA +
       
   527   options [document = false]
   518   theories DBuffer
   528   theories DBuffer
   519 
   529 
   520 session Memory in "TLA/Memory" = TLA +
   530 session Memory in "TLA/Memory" = TLA +
       
   531   options [document = false]
   521   theories MemoryImplementation
   532   theories MemoryImplementation
   522 
   533 
   523 session TPTP = HOL +
   534 session TPTP = HOL +
   524   description {*
   535   description {*
   525     Author:     Jasmin Blanchette, TU Muenchen
   536     Author:     Jasmin Blanchette, TU Muenchen
   526     Author:     Nik Sultana, University of Cambridge
   537     Author:     Nik Sultana, University of Cambridge
   527     Copyright   2011
   538     Copyright   2011
   528 
   539 
   529     TPTP-related extensions.
   540     TPTP-related extensions.
   530   *}
   541   *}
       
   542   options [document = false]
   531   theories
   543   theories
   532     ATP_Theory_Export
   544     ATP_Theory_Export
   533     MaSh_Eval
   545     MaSh_Eval
   534     MaSh_Export
   546     MaSh_Export
   535     TPTP_Interpret
   547     TPTP_Interpret
   557     "ex/Dining_Cryptographers"
   569     "ex/Dining_Cryptographers"
   558     "ex/Koepf_Duermuth_Countermeasure"
   570     "ex/Koepf_Duermuth_Countermeasure"
   559   files "document/root.tex"
   571   files "document/root.tex"
   560 
   572 
   561 session Nominal = HOL +
   573 session Nominal = HOL +
       
   574   options [document = false]
   562   theories Nominal
   575   theories Nominal
   563 
   576 
   564 session Examples in "Nominal/Examples" = "HOL-Nominal" +
   577 session Examples in "Nominal/Examples" = "HOL-Nominal" +
       
   578   options [document = false]
   565   theories Nominal_Examples
   579   theories Nominal_Examples
   566   theories [quick_and_dirty] VC_Condition
   580   theories [quick_and_dirty] VC_Condition
   567 
   581 
   568 session Word = HOL +
   582 session Word = HOL +
   569   options [document_graph]
   583   options [document_graph]
   570   theories Word
   584   theories Word
   571   files "document/root.bib" "document/root.tex"
   585   files "document/root.bib" "document/root.tex"
   572 
   586 
   573 session Examples in "Word/Examples" = "HOL-Word" +
   587 session Examples in "Word/Examples" = "HOL-Word" +
       
   588   options [document = false]
   574   theories WordExamples
   589   theories WordExamples
   575 
   590 
   576 session Statespace = HOL +
   591 session Statespace = HOL +
   577   theories StateSpaceEx
   592   theories StateSpaceEx
   578   files "document/root.tex"
   593   files "document/root.tex"
   581   options [document_graph]
   596   options [document_graph]
   582   theories Hypercomplex
   597   theories Hypercomplex
   583   files "document/root.tex"
   598   files "document/root.tex"
   584 
   599 
   585 session Examples in "NSA/Examples" = "HOL-NSA" +
   600 session Examples in "NSA/Examples" = "HOL-NSA" +
       
   601   options [document = false]
   586   theories NSPrimes
   602   theories NSPrimes
   587 
   603 
   588 session Mirabelle = HOL +
   604 session Mirabelle = HOL +
       
   605   options [document = false]
   589   theories Mirabelle_Test
   606   theories Mirabelle_Test
   590 (* FIXME
   607 (* FIXME
   591 	@cd Library; $(ISABELLE_TOOL) mirabelle -q arith Inner_Product.thy # some arbitrary small test case
   608 	@cd Library; $(ISABELLE_TOOL) mirabelle -q arith Inner_Product.thy # some arbitrary small test case
   592 *)
   609 *)
   593 
   610 
   594 session SMT_Examples = "HOL-Word" +
   611 session SMT_Examples = "HOL-Word" +
   595   options [quick_and_dirty]
   612   options [document = false, quick_and_dirty]
   596   theories
   613   theories
   597     SMT_Tests
   614     SMT_Tests
   598     SMT_Examples
   615     SMT_Examples
   599     SMT_Word_Examples
   616     SMT_Word_Examples
   600   files
   617   files
   601     "SMT_Examples.certs"
   618     "SMT_Examples.certs"
   602     "SMT_Tests.certs"
   619     "SMT_Tests.certs"
   603 
   620 
   604 session "HOL-Boogie"! in "Boogie" = "HOL-Word" +
   621 session "HOL-Boogie"! in "Boogie" = "HOL-Word" +
       
   622   options [document = false]
   605   theories Boogie
   623   theories Boogie
   606   (* FIXME files!?! *)
   624   (* FIXME files!?! *)
   607 
   625 
   608 session Examples in "Boogie/Examples" = "HOL-Boogie" +
   626 session Examples in "Boogie/Examples" = "HOL-Boogie" +
       
   627   options [document = false]
   609   theories
   628   theories
   610     Boogie_Max_Stepwise
   629     Boogie_Max_Stepwise
   611     Boogie_Max
   630     Boogie_Max
   612     Boogie_Dijkstra
   631     Boogie_Dijkstra
   613     VCC_Max
   632     VCC_Max
   615     "Boogie_Dijkstra.certs"
   634     "Boogie_Dijkstra.certs"
   616     "Boogie_Max.certs"
   635     "Boogie_Max.certs"
   617     "VCC_Max.certs"
   636     "VCC_Max.certs"
   618 
   637 
   619 session "HOL-SPARK"! in "SPARK" = "HOL-Word" +
   638 session "HOL-SPARK"! in "SPARK" = "HOL-Word" +
       
   639   options [document = false]
   620   theories SPARK
   640   theories SPARK
   621 
   641 
   622 session Examples in "SPARK/Examples" = "HOL-SPARK" +
   642 session Examples in "SPARK/Examples" = "HOL-SPARK" +
       
   643   options [document = false]
   623   theories
   644   theories
   624     "Gcd/Greatest_Common_Divisor"
   645     "Gcd/Greatest_Common_Divisor"
   625 
   646 
   626     "Liseq/Longest_Increasing_Subsequence"
   647     "Liseq/Longest_Increasing_Subsequence"
   627 
   648 
   703     "simple_greatest_common_divisor/g_c_d.fdl"
   724     "simple_greatest_common_divisor/g_c_d.fdl"
   704     "simple_greatest_common_divisor/g_c_d.rls"
   725     "simple_greatest_common_divisor/g_c_d.rls"
   705     "simple_greatest_common_divisor/g_c_d.siv"
   726     "simple_greatest_common_divisor/g_c_d.siv"
   706 
   727 
   707 session Mutabelle = HOL +
   728 session Mutabelle = HOL +
       
   729   options [document = false]
   708   theories MutabelleExtra
   730   theories MutabelleExtra
   709 
   731 
   710 session Quickcheck_Examples = HOL +
   732 session Quickcheck_Examples = HOL +
       
   733   options [document = false]
   711   theories Quickcheck_Examples  (* FIXME *)
   734   theories Quickcheck_Examples  (* FIXME *)
   712 
   735 
   713 session Quotient_Examples = HOL +
   736 session Quotient_Examples = HOL +
   714   description {*
   737   description {*
   715     Author:     Cezary Kaliszyk and Christian Urban
   738     Author:     Cezary Kaliszyk and Christian Urban
   716   *}
   739   *}
       
   740   options [document = false]
   717   theories
   741   theories
   718     DList
   742     DList
   719     FSet
   743     FSet
   720     Quotient_Int
   744     Quotient_Int
   721     Quotient_Message
   745     Quotient_Message
   725     Lift_Fun
   749     Lift_Fun
   726     Quotient_Rat
   750     Quotient_Rat
   727     Lift_DList
   751     Lift_DList
   728 
   752 
   729 session Predicate_Compile_Examples = HOL +
   753 session Predicate_Compile_Examples = HOL +
       
   754   options [document = false]
   730   theories  (* FIXME *)
   755   theories  (* FIXME *)
   731     Examples
   756     Examples
   732     Predicate_Compile_Tests
   757     Predicate_Compile_Tests
   733     Specialisation_Examples
   758     Specialisation_Examples
   734 
   759 
   755     Fixrec_ex
   780     Fixrec_ex
   756     New_Domain
   781     New_Domain
   757   files "document/root.tex"
   782   files "document/root.tex"
   758 
   783 
   759 session Library in "HOLCF/Library" = HOLCF +
   784 session Library in "HOLCF/Library" = HOLCF +
       
   785   options [document = false]
   760   theories HOLCF_Library
   786   theories HOLCF_Library
   761 
   787 
   762 session IMP in "HOLCF/IMP" = HOLCF +
   788 session IMP in "HOLCF/IMP" = HOLCF +
       
   789   options [document = false]
   763   theories HoareEx
   790   theories HoareEx
   764   files "document/root.tex"
   791   files "document/root.tex"
   765 
   792 
   766 session ex in "HOLCF/ex" = HOLCF +
   793 session ex in "HOLCF/ex" = HOLCF +
   767   description {* Misc HOLCF examples *}
   794   description {* Misc HOLCF examples *}
       
   795   options [document = false]
   768   theories
   796   theories
   769     Dnat
   797     Dnat
   770     Dagstuhl
   798     Dagstuhl
   771     Focus_ex
   799     Focus_ex
   772     Fix2
   800     Fix2
   777     Domain_Proofs
   805     Domain_Proofs
   778     Letrec
   806     Letrec
   779     Pattern_Match
   807     Pattern_Match
   780 
   808 
   781 session FOCUS in "HOLCF/FOCUS" = HOLCF +
   809 session FOCUS in "HOLCF/FOCUS" = HOLCF +
       
   810   options [document = false]
   782   theories
   811   theories
   783     Fstreams
   812     Fstreams
   784     FOCUS
   813     FOCUS
   785     Buffer_adm
   814     Buffer_adm
   786 
   815 
   788   description {*
   817   description {*
   789     Author:     Olaf Mueller
   818     Author:     Olaf Mueller
   790 
   819 
   791     Formalization of a semantic model of I/O-Automata.
   820     Formalization of a semantic model of I/O-Automata.
   792   *}
   821   *}
       
   822   options [document = false]
   793   theories "meta_theory/Abstraction"
   823   theories "meta_theory/Abstraction"
   794 
   824 
   795 session ABP in "HOLCF/IOA/ABP" = IOA +
   825 session ABP in "HOLCF/IOA/ABP" = IOA +
   796   description {*
   826   description {*
   797     Author:     Olaf Mueller
   827     Author:     Olaf Mueller
   798 
   828 
   799     The Alternating Bit Protocol performed in I/O-Automata.
   829     The Alternating Bit Protocol performed in I/O-Automata.
   800   *}
   830   *}
       
   831   options [document = false]
   801   theories Correctness
   832   theories Correctness
   802 
   833 
   803 session NTP in "HOLCF/IOA/NTP" = IOA +
   834 session NTP in "HOLCF/IOA/NTP" = IOA +
   804   description {*
   835   description {*
   805     Author:     Tobias Nipkow & Konrad Slind
   836     Author:     Tobias Nipkow & Konrad Slind
   806 
   837 
   807     A network transmission protocol, performed in the
   838     A network transmission protocol, performed in the
   808     I/O automata formalization by Olaf Mueller.
   839     I/O automata formalization by Olaf Mueller.
   809   *}
   840   *}
       
   841   options [document = false]
   810   theories Correctness
   842   theories Correctness
   811 
   843 
   812 session Storage in "HOLCF/IOA/Storage" = IOA +
   844 session Storage in "HOLCF/IOA/Storage" = IOA +
   813   description {*
   845   description {*
   814     Author:     Olaf Mueller
   846     Author:     Olaf Mueller
   815 
   847 
   816     Memory storage case study.
   848     Memory storage case study.
   817   *}
   849   *}
       
   850   options [document = false]
   818   theories Correctness
   851   theories Correctness
   819 
   852 
   820 session ex in "HOLCF/IOA/ex" = IOA +
   853 session ex in "HOLCF/IOA/ex" = IOA +
   821   description {*
   854   description {*
   822     Author:     Olaf Mueller
   855     Author:     Olaf Mueller
   823   *}
   856   *}
       
   857   options [document = false]
   824   theories
   858   theories
   825     TrivEx
   859     TrivEx
   826     TrivEx2
   860     TrivEx2
   827 
   861 
   828 session Datatype_Benchmark = HOL +
   862 session Datatype_Benchmark = HOL +
   829   description {* Some rather large datatype examples (from John Harrison). *}
   863   description {* Some rather large datatype examples (from John Harrison). *}
       
   864   options [document = false]
   830   theories [condition = ISABELLE_BENCHMARK]
   865   theories [condition = ISABELLE_BENCHMARK]
   831     (* FIXME Toplevel.timing := true; *)
   866     (* FIXME Toplevel.timing := true; *)
   832     Brackin
   867     Brackin
   833     Instructions
   868     Instructions
   834     SML
   869     SML
   835     Verilog
   870     Verilog
   836 
   871 
   837 session Record_Benchmark = HOL +
   872 session Record_Benchmark = HOL +
   838   description {* Some benchmark on large record. *}
   873   description {* Some benchmark on large record. *}
       
   874   options [document = false]
   839   theories [condition = ISABELLE_BENCHMARK]
   875   theories [condition = ISABELLE_BENCHMARK]
   840     (* FIXME Toplevel.timing := true; *)
   876     (* FIXME Toplevel.timing := true; *)
   841     Record_Benchmark
   877     Record_Benchmark
   842 
   878 
   843