src/HOL/ROOT
changeset 65543 8369b33fda0a
parent 65538 a39ef48fbee0
child 65544 c09c11386ca5
equal deleted inserted replaced
65542:6a00518bbfcc 65543:8369b33fda0a
    18   description {*
    18   description {*
    19     HOL-Main with explicit proof terms.
    19     HOL-Main with explicit proof terms.
    20   *}
    20   *}
    21   options [document = false, theory_qualifier = "HOL",
    21   options [document = false, theory_qualifier = "HOL",
    22     quick_and_dirty = false, record_proofs = 2, parallel_proofs = 0]
    22     quick_and_dirty = false, record_proofs = 2, parallel_proofs = 0]
    23   sessions "HOL-Library"
    23   sessions
       
    24     "HOL-Library"
    24   theories
    25   theories
    25     GCD
    26     GCD
    26     Binomial
    27     Binomial
    27     "HOL-Library.Old_Datatype"
    28     "HOL-Library.Old_Datatype"
    28   files
    29   files
    61     Old_SMT
    62     Old_SMT
    62     Refute
    63     Refute
    63   document_files "root.bib" "root.tex"
    64   document_files "root.bib" "root.tex"
    64 
    65 
    65 session "HOL-Analysis" (main timing) in Analysis = HOL +
    66 session "HOL-Analysis" (main timing) in Analysis = HOL +
       
    67   sessions
       
    68     "HOL-Library"
       
    69     "HOL-Computational_Algebra"
    66   theories
    70   theories
    67     Analysis
    71     Analysis
    68   document_files
    72   document_files
    69     "root.tex"
    73     "root.tex"
    70 
    74 
    72   theories
    76   theories
    73     Approximations
    77     Approximations
    74     Circle_Area
    78     Circle_Area
    75 
    79 
    76 session "HOL-Computational_Algebra" in "Computational_Algebra" = HOL +
    80 session "HOL-Computational_Algebra" in "Computational_Algebra" = HOL +
       
    81   sessions
       
    82     "HOL-Library"
    77   theories
    83   theories
    78     Computational_Algebra
    84     Computational_Algebra
    79     (*conflicting type class instantiations and dependent applications*)
    85     (*conflicting type class instantiations and dependent applications*)
    80     Field_as_Ring
    86     Field_as_Ring
    81     Polynomial_Factorial
    87     Polynomial_Factorial
    96 
   102 
    97     The theorem says, that every continous linearform, defined on arbitrary
   103     The theorem says, that every continous linearform, defined on arbitrary
    98     subspaces (not only one-dimensional subspaces), can be extended to a
   104     subspaces (not only one-dimensional subspaces), can be extended to a
    99     continous linearform on the whole vectorspace.
   105     continous linearform on the whole vectorspace.
   100   *}
   106   *}
   101   theories Hahn_Banach
   107   sessions
       
   108     "HOL-Library"
       
   109   theories
       
   110     Hahn_Banach
   102   document_files "root.bib" "root.tex"
   111   document_files "root.bib" "root.tex"
   103 
   112 
   104 session "HOL-Induct" in Induct = HOL +
   113 session "HOL-Induct" in Induct = HOL +
   105   description {*
   114   description {*
   106     Examples of (Co)Inductive Definitions.
   115     Examples of (Co)Inductive Definitions.
   116     http://www.cl.cam.ac.uk/Research/Reports/TR312-lcp-set-II.ps.gz).
   125     http://www.cl.cam.ac.uk/Research/Reports/TR312-lcp-set-II.ps.gz).
   117 
   126 
   118     Exp demonstrates the use of iterated inductive definitions to reason about
   127     Exp demonstrates the use of iterated inductive definitions to reason about
   119     mutually recursive relations.
   128     mutually recursive relations.
   120   *}
   129   *}
       
   130   sessions
       
   131     "HOL-Library"
   121   theories [document = false]
   132   theories [document = false]
   122     "~~/src/HOL/Library/Old_Datatype"
   133     "~~/src/HOL/Library/Old_Datatype"
   123   theories [quick_and_dirty]
   134   theories [quick_and_dirty]
   124     Common_Patterns
   135     Common_Patterns
   125   theories
   136   theories
   217 session "HOL-Number_Theory" (timing) in Number_Theory = HOL +
   228 session "HOL-Number_Theory" (timing) in Number_Theory = HOL +
   218   description {*
   229   description {*
   219     Fundamental Theorem of Arithmetic, Chinese Remainder Theorem, Fermat/Euler
   230     Fundamental Theorem of Arithmetic, Chinese Remainder Theorem, Fermat/Euler
   220     Theorem, Wilson's Theorem, some lemmas for Quadratic Reciprocity.
   231     Theorem, Wilson's Theorem, some lemmas for Quadratic Reciprocity.
   221   *}
   232   *}
       
   233   sessions
       
   234     "HOL-Library"
       
   235     "HOL-Algebra"
       
   236     "HOL-Computational_Algebra"
   222   theories [document = false]
   237   theories [document = false]
   223     "~~/src/HOL/Library/FuncSet"
   238     "~~/src/HOL/Library/FuncSet"
   224     "~~/src/HOL/Library/Multiset"
   239     "~~/src/HOL/Library/Multiset"
   225     "~~/src/HOL/Algebra/Ring"
   240     "~~/src/HOL/Algebra/Ring"
   226     "~~/src/HOL/Algebra/FiniteProduct"
   241     "~~/src/HOL/Algebra/FiniteProduct"
   245   theories Hoare_Parallel
   260   theories Hoare_Parallel
   246   document_files "root.bib" "root.tex"
   261   document_files "root.bib" "root.tex"
   247 
   262 
   248 session "HOL-Codegenerator_Test" in Codegenerator_Test = "HOL-Library" +
   263 session "HOL-Codegenerator_Test" in Codegenerator_Test = "HOL-Library" +
   249   options [document = false, browser_info = false]
   264   options [document = false, browser_info = false]
       
   265   sessions
       
   266     "HOL-Computational_Algebra"
       
   267     "HOL-Number_Theory"
   250   theories
   268   theories
   251     Generate
   269     Generate
   252     Generate_Binary_Nat
   270     Generate_Binary_Nat
   253     Generate_Target_Nat
   271     Generate_Target_Nat
   254     Generate_Efficient_Datastructures
   272     Generate_Efficient_Datastructures
   305   description {*
   323   description {*
   306     Author: Clemens Ballarin, started 24 September 1999
   324     Author: Clemens Ballarin, started 24 September 1999
   307 
   325 
   308     The Isabelle Algebraic Library.
   326     The Isabelle Algebraic Library.
   309   *}
   327   *}
       
   328   sessions
       
   329     "HOL-Library"
       
   330     "HOL-Computational_Algebra"
   310   theories [document = false]
   331   theories [document = false]
   311     (* Preliminaries from set and number theory *)
   332     (* Preliminaries from set and number theory *)
   312     "~~/src/HOL/Library/FuncSet"
   333     "~~/src/HOL/Library/FuncSet"
   313     "~~/src/HOL/Computational_Algebra/Primes"
   334     "~~/src/HOL/Computational_Algebra/Primes"
   314     "~~/src/HOL/Library/Permutation"
   335     "~~/src/HOL/Library/Permutation"
   396   theories MainZF Games
   417   theories MainZF Games
   397   document_files "root.tex"
   418   document_files "root.tex"
   398 
   419 
   399 session "HOL-Imperative_HOL" in Imperative_HOL = HOL +
   420 session "HOL-Imperative_HOL" in Imperative_HOL = HOL +
   400   options [print_mode = "iff,no_brackets"]
   421   options [print_mode = "iff,no_brackets"]
       
   422   sessions
       
   423     "HOL-Library"
   401   theories [document = false]
   424   theories [document = false]
   402     "~~/src/HOL/Library/Countable"
   425     "~~/src/HOL/Library/Countable"
   403     "~~/src/HOL/Library/Monad_Syntax"
   426     "~~/src/HOL/Library/Monad_Syntax"
   404     "~~/src/HOL/Library/LaTeXsugar"
   427     "~~/src/HOL/Library/LaTeXsugar"
   405   theories Imperative_HOL_ex
   428   theories Imperative_HOL_ex
   408 session "HOL-Decision_Procs" (timing) in Decision_Procs = HOL +
   431 session "HOL-Decision_Procs" (timing) in Decision_Procs = HOL +
   409   description {*
   432   description {*
   410     Various decision procedures, typically involving reflection.
   433     Various decision procedures, typically involving reflection.
   411   *}
   434   *}
   412   options [document = false]
   435   options [document = false]
   413   theories Decision_Procs
   436   sessions
       
   437     "HOL-Library"
       
   438     "HOL-Algebra"
       
   439   theories
       
   440     Decision_Procs
   414 
   441 
   415 session "HOL-Proofs-ex" in "Proofs/ex" = "HOL-Proofs" +
   442 session "HOL-Proofs-ex" in "Proofs/ex" = "HOL-Proofs" +
   416   options [document = false]
   443   options [document = false]
   417   theories
   444   theories
   418     Hilbert_Classical
   445     Hilbert_Classical
   422 session "HOL-Proofs-Extraction" (timing) in "Proofs/Extraction" = "HOL-Proofs" +
   449 session "HOL-Proofs-Extraction" (timing) in "Proofs/Extraction" = "HOL-Proofs" +
   423   description {*
   450   description {*
   424     Examples for program extraction in Higher-Order Logic.
   451     Examples for program extraction in Higher-Order Logic.
   425   *}
   452   *}
   426   options [parallel_proofs = 0, quick_and_dirty = false]
   453   options [parallel_proofs = 0, quick_and_dirty = false]
       
   454   sessions
       
   455     "HOL-Library"
       
   456     "HOL-Computational_Algebra"
   427   theories [document = false]
   457   theories [document = false]
   428     "~~/src/HOL/Library/Code_Target_Numeral"
   458     "~~/src/HOL/Library/Code_Target_Numeral"
   429     "~~/src/HOL/Library/Monad_Syntax"
   459     "~~/src/HOL/Library/Monad_Syntax"
   430     "~~/src/HOL/Computational_Algebra/Primes"
   460     "~~/src/HOL/Computational_Algebra/Primes"
   431     "~~/src/HOL/Library/State_Monad"
   461     "~~/src/HOL/Library/State_Monad"
   447     The paper "More Church-Rosser Proofs (in Isabelle/HOL)" describes the whole
   477     The paper "More Church-Rosser Proofs (in Isabelle/HOL)" describes the whole
   448     theory (see http://www.in.tum.de/~nipkow/pubs/jar2001.html).
   478     theory (see http://www.in.tum.de/~nipkow/pubs/jar2001.html).
   449   *}
   479   *}
   450   options [print_mode = "no_brackets",
   480   options [print_mode = "no_brackets",
   451     parallel_proofs = 0, quick_and_dirty = false]
   481     parallel_proofs = 0, quick_and_dirty = false]
   452   sessions "HOL-Library"
   482   sessions
       
   483     "HOL-Library"
   453   theories
   484   theories
   454     Eta
   485     Eta
   455     StrongNorm
   486     StrongNorm
   456     Standardization
   487     Standardization
   457     WeakNorm
   488     WeakNorm
   474   description {*
   505   description {*
   475     Formalization of a fragment of Java, together with a corresponding virtual
   506     Formalization of a fragment of Java, together with a corresponding virtual
   476     machine and a specification of its bytecode verifier and a lightweight
   507     machine and a specification of its bytecode verifier and a lightweight
   477     bytecode verifier, including proofs of type-safety.
   508     bytecode verifier, including proofs of type-safety.
   478   *}
   509   *}
       
   510   sessions
       
   511     "HOL-Library"
   479   theories [document = false]
   512   theories [document = false]
   480     "~~/src/HOL/Library/While_Combinator"
   513     "~~/src/HOL/Library/While_Combinator"
   481   theories
   514   theories
   482     MicroJava
   515     MicroJava
   483   document_files
   516   document_files
   543 
   576 
   544 session "HOL-ex" in ex = HOL +
   577 session "HOL-ex" in ex = HOL +
   545   description {*
   578   description {*
   546     Miscellaneous examples for Higher-Order Logic.
   579     Miscellaneous examples for Higher-Order Logic.
   547   *}
   580   *}
       
   581   sessions
       
   582     "HOL-Library"
       
   583     "HOL-Number_Theory"
   548   theories [document = false]
   584   theories [document = false]
   549     "~~/src/HOL/Library/State_Monad"
   585     "~~/src/HOL/Library/State_Monad"
   550     Code_Binary_Nat_examples
   586     Code_Binary_Nat_examples
   551     "~~/src/HOL/Library/FuncSet"
   587     "~~/src/HOL/Library/FuncSet"
   552     Eval_Examples
   588     Eval_Examples
   639 session "HOL-Isar_Examples" in Isar_Examples = HOL +
   675 session "HOL-Isar_Examples" in Isar_Examples = HOL +
   640   description {*
   676   description {*
   641     Miscellaneous Isabelle/Isar examples.
   677     Miscellaneous Isabelle/Isar examples.
   642   *}
   678   *}
   643   options [quick_and_dirty]
   679   options [quick_and_dirty]
       
   680   sessions
       
   681     "HOL-Library"
       
   682     "HOL-Computational_Algebra"
   644   theories [document = false]
   683   theories [document = false]
   645     "~~/src/HOL/Library/Lattice_Syntax"
   684     "~~/src/HOL/Library/Lattice_Syntax"
   646     "../Computational_Algebra/Primes"
   685     "../Computational_Algebra/Primes"
   647   theories
   686   theories
   648     Knaster_Tarski
   687     Knaster_Tarski
   678 
   717 
   679 session "HOL-SET_Protocol" (timing) in SET_Protocol = HOL +
   718 session "HOL-SET_Protocol" (timing) in SET_Protocol = HOL +
   680   description {*
   719   description {*
   681     Verification of the SET Protocol.
   720     Verification of the SET Protocol.
   682   *}
   721   *}
   683   theories [document = false] "~~/src/HOL/Library/Nat_Bijection"
   722   sessions
   684   theories SET_Protocol
   723     "HOL-Library"
       
   724   theories [document = false]
       
   725     "~~/src/HOL/Library/Nat_Bijection"
       
   726   theories
       
   727     SET_Protocol
   685   document_files "root.tex"
   728   document_files "root.tex"
   686 
   729 
   687 session "HOL-Matrix_LP" in Matrix_LP = HOL +
   730 session "HOL-Matrix_LP" in Matrix_LP = HOL +
   688   description {*
   731   description {*
   689     Two-dimensional matrices and linear programming.
   732     Two-dimensional matrices and linear programming.
   727     TPTP_Proof_Reconstruction
   770     TPTP_Proof_Reconstruction
   728   theories
   771   theories
   729     ATP_Problem_Import
   772     ATP_Problem_Import
   730 
   773 
   731 session "HOL-Probability" (main timing) in "Probability" = "HOL-Analysis" +
   774 session "HOL-Probability" (main timing) in "Probability" = "HOL-Analysis" +
       
   775   sessions
       
   776     "HOL-Library"
   732   theories [document = false]
   777   theories [document = false]
   733     "~~/src/HOL/Library/Countable"
   778     "~~/src/HOL/Library/Countable"
   734     "~~/src/HOL/Library/Permutation"
   779     "~~/src/HOL/Library/Permutation"
   735     "~~/src/HOL/Library/Order_Continuity"
   780     "~~/src/HOL/Library/Order_Continuity"
   736     "~~/src/HOL/Library/Diagonal_Subsequence"
   781     "~~/src/HOL/Library/Diagonal_Subsequence"
   853     Nonstandard_Analysis
   898     Nonstandard_Analysis
   854   document_files "root.tex"
   899   document_files "root.tex"
   855 
   900 
   856 session "HOL-Nonstandard_Analysis-Examples" (timing) in "Nonstandard_Analysis/Examples" = "HOL-Nonstandard_Analysis" +
   901 session "HOL-Nonstandard_Analysis-Examples" (timing) in "Nonstandard_Analysis/Examples" = "HOL-Nonstandard_Analysis" +
   857   options [document = false]
   902   options [document = false]
   858   theories NSPrimes
   903   sessions
       
   904     "HOL-Computational_Algebra"
       
   905   theories
       
   906     NSPrimes
   859 
   907 
   860 session "HOL-Mirabelle" in Mirabelle = HOL +
   908 session "HOL-Mirabelle" in Mirabelle = HOL +
   861   options [document = false]
   909   options [document = false]
   862   theories Mirabelle_Test
   910   theories Mirabelle_Test
   863 
   911 
   990 session "HOL-Quotient_Examples" (timing) in Quotient_Examples = HOL +
  1038 session "HOL-Quotient_Examples" (timing) in Quotient_Examples = HOL +
   991   description {*
  1039   description {*
   992     Author:     Cezary Kaliszyk and Christian Urban
  1040     Author:     Cezary Kaliszyk and Christian Urban
   993   *}
  1041   *}
   994   options [document = false]
  1042   options [document = false]
       
  1043   sessions
       
  1044     "HOL-Library"
   995   theories
  1045   theories
   996     DList
  1046     DList
   997     Quotient_FSet
  1047     Quotient_FSet
   998     Quotient_Int
  1048     Quotient_Int
   999     Quotient_Message
  1049     Quotient_Message
  1043     Author:     Franz Regensburger
  1093     Author:     Franz Regensburger
  1044     Author:     Brian Huffman
  1094     Author:     Brian Huffman
  1045 
  1095 
  1046     HOLCF -- a semantic extension of HOL by the LCF logic.
  1096     HOLCF -- a semantic extension of HOL by the LCF logic.
  1047   *}
  1097   *}
       
  1098   sessions
       
  1099     "HOL-Library"
  1048   theories [document = false]
  1100   theories [document = false]
  1049     "~~/src/HOL/Library/Nat_Bijection"
  1101     "~~/src/HOL/Library/Nat_Bijection"
  1050     "~~/src/HOL/Library/Countable"
  1102     "~~/src/HOL/Library/Countable"
  1051   theories
  1103   theories
  1052     HOLCF (global)
  1104     HOLCF (global)