src/HOL/ROOT
changeset 62357 ab76bd43c14a
parent 62352 35a9e1cbb5b3
parent 62354 fdd6989cc8a0
child 62363 7b5468422352
equal deleted inserted replaced
62353:7f927120b5a2 62357:ab76bd43c14a
    16 
    16 
    17 session "HOL-Proofs" (slow) = Pure +
    17 session "HOL-Proofs" (slow) = Pure +
    18   description {*
    18   description {*
    19     HOL-Main with explicit proof terms.
    19     HOL-Main with explicit proof terms.
    20   *}
    20   *}
    21   options [condition = ML_SYSTEM_POLYML, 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!*)
    23   theories "~~/src/HOL/Library/Old_Datatype"
    23   theories "~~/src/HOL/Library/Old_Datatype"
    24   files
    24   files
    25     "Tools/Quickcheck/Narrowing_Engine.hs"
    25     "Tools/Quickcheck/Narrowing_Engine.hs"
    26     "Tools/Quickcheck/PNF_Narrowing_Engine.hs"
    26     "Tools/Quickcheck/PNF_Narrowing_Engine.hs"
   244   *}
   244   *}
   245   theories Hoare_Parallel
   245   theories Hoare_Parallel
   246   document_files "root.bib" "root.tex"
   246   document_files "root.bib" "root.tex"
   247 
   247 
   248 session "HOL-Codegenerator_Test" in Codegenerator_Test = "HOL-Library" +
   248 session "HOL-Codegenerator_Test" in Codegenerator_Test = "HOL-Library" +
   249   options [condition = ML_SYSTEM_POLYML, document = false, browser_info = false]
   249   options [document = false, browser_info = false]
   250   theories
   250   theories
   251     Generate
   251     Generate
   252     Generate_Binary_Nat
   252     Generate_Binary_Nat
   253     Generate_Target_Nat
   253     Generate_Target_Nat
   254     Generate_Efficient_Datastructures
   254     Generate_Efficient_Datastructures
   255     Generate_Pretty_Char
   255     Generate_Pretty_Char
   256   theories [condition = "ML_SYSTEM_POLYML,ISABELLE_GHC"]
   256   theories [condition = "ISABELLE_GHC"]
   257     Code_Test_GHC
   257     Code_Test_GHC
   258   theories [condition = "ML_SYSTEM_POLYML,ISABELLE_MLTON"]
   258   theories [condition = "ISABELLE_MLTON"]
   259     Code_Test_MLton
   259     Code_Test_MLton
   260   theories [condition = "ML_SYSTEM_POLYML,ISABELLE_OCAMLC"]
   260   theories [condition = "ISABELLE_OCAMLC"]
   261     Code_Test_OCaml
   261     Code_Test_OCaml
   262   theories [condition = "ML_SYSTEM_POLYML,ISABELLE_POLYML"]
   262   theories [condition = "ISABELLE_POLYML"]
   263     Code_Test_PolyML
   263     Code_Test_PolyML
   264   theories [condition = "ML_SYSTEM_POLYML,ISABELLE_SCALA"]
   264   theories [condition = "ISABELLE_SCALA"]
   265     Code_Test_Scala
   265     Code_Test_Scala
   266   theories [condition = "ML_SYSTEM_POLYML,ISABELLE_SMLNJ"]
   266   theories [condition = "ISABELLE_SMLNJ"]
   267     Code_Test_SMLNJ
   267     Code_Test_SMLNJ
   268 
   268 
   269 session "HOL-Metis_Examples" in Metis_Examples = HOL +
   269 session "HOL-Metis_Examples" in Metis_Examples = HOL +
   270   description {*
   270   description {*
   271     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
   271     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
   393 
   393 
   394 session "HOL-Decision_Procs" in Decision_Procs = HOL +
   394 session "HOL-Decision_Procs" in Decision_Procs = HOL +
   395   description {*
   395   description {*
   396     Various decision procedures, typically involving reflection.
   396     Various decision procedures, typically involving reflection.
   397   *}
   397   *}
   398   options [condition = ML_SYSTEM_POLYML, document = false]
   398   options [document = false]
   399   theories Decision_Procs
   399   theories Decision_Procs
   400 
   400 
   401 session "HOL-Proofs-ex" in "Proofs/ex" = "HOL-Proofs" +
   401 session "HOL-Proofs-ex" in "Proofs/ex" = "HOL-Proofs" +
   402   options [condition = ML_SYSTEM_POLYML, document = false, parallel_proofs = 0]
   402   options [document = false, parallel_proofs = 0]
   403   theories
   403   theories
   404     Hilbert_Classical
   404     Hilbert_Classical
   405     XML_Data
   405     XML_Data
   406 
   406 
   407 session "HOL-Proofs-Extraction" in "Proofs/Extraction" = "HOL-Proofs" +
   407 session "HOL-Proofs-Extraction" in "Proofs/Extraction" = "HOL-Proofs" +
   408   description {*
   408   description {*
   409     Examples for program extraction in Higher-Order Logic.
   409     Examples for program extraction in Higher-Order Logic.
   410   *}
   410   *}
   411   options [condition = ML_SYSTEM_POLYML, parallel_proofs = 0, quick_and_dirty = false]
   411   options [parallel_proofs = 0, quick_and_dirty = false]
   412   theories [document = false]
   412   theories [document = false]
   413     "~~/src/HOL/Library/Code_Target_Numeral"
   413     "~~/src/HOL/Library/Code_Target_Numeral"
   414     "~~/src/HOL/Library/Monad_Syntax"
   414     "~~/src/HOL/Library/Monad_Syntax"
   415     "~~/src/HOL/Number_Theory/Primes"
   415     "~~/src/HOL/Number_Theory/Primes"
   416     "~~/src/HOL/Number_Theory/UniqueFactorization"
   416     "~~/src/HOL/Number_Theory/UniqueFactorization"
   431     proves confluence of beta, eta and beta+eta.
   431     proves confluence of beta, eta and beta+eta.
   432 
   432 
   433     The paper "More Church-Rosser Proofs (in Isabelle/HOL)" describes the whole
   433     The paper "More Church-Rosser Proofs (in Isabelle/HOL)" describes the whole
   434     theory (see http://www.in.tum.de/~nipkow/pubs/jar2001.html).
   434     theory (see http://www.in.tum.de/~nipkow/pubs/jar2001.html).
   435   *}
   435   *}
   436   options [condition = ML_SYSTEM_POLYML, print_mode = "no_brackets",
   436   options [print_mode = "no_brackets",
   437     parallel_proofs = 0, quick_and_dirty = false]
   437     parallel_proofs = 0, quick_and_dirty = false]
   438   theories [document = false]
   438   theories [document = false]
   439     "~~/src/HOL/Library/Code_Target_Int"
   439     "~~/src/HOL/Library/Code_Target_Int"
   440   theories
   440   theories
   441     Eta
   441     Eta
   530 
   530 
   531 session "HOL-ex" in ex = HOL +
   531 session "HOL-ex" in ex = HOL +
   532   description {*
   532   description {*
   533     Miscellaneous examples for Higher-Order Logic.
   533     Miscellaneous examples for Higher-Order Logic.
   534   *}
   534   *}
   535   options [condition = ML_SYSTEM_POLYML]
       
   536   theories [document = false]
   535   theories [document = false]
   537     "~~/src/HOL/Library/State_Monad"
   536     "~~/src/HOL/Library/State_Monad"
   538     Code_Binary_Nat_examples
   537     Code_Binary_Nat_examples
   539     "~~/src/HOL/Library/FuncSet"
   538     "~~/src/HOL/Library/FuncSet"
   540     Eval_Examples
   539     Eval_Examples
   701     Author:     Nik Sultana, University of Cambridge
   700     Author:     Nik Sultana, University of Cambridge
   702     Copyright   2011
   701     Copyright   2011
   703 
   702 
   704     TPTP-related extensions.
   703     TPTP-related extensions.
   705   *}
   704   *}
   706   options [condition = ML_SYSTEM_POLYML, document = false]
   705   options [document = false]
   707   theories
   706   theories
   708     ATP_Theory_Export
   707     ATP_Theory_Export
   709     MaSh_Eval
   708     MaSh_Eval
   710     TPTP_Interpret
   709     TPTP_Interpret
   711     THF_Arith
   710     THF_Arith
   747 session "HOL-Nominal" in Nominal = HOL +
   746 session "HOL-Nominal" in Nominal = HOL +
   748   options [document = false]
   747   options [document = false]
   749   theories Nominal
   748   theories Nominal
   750 
   749 
   751 session "HOL-Nominal-Examples" in "Nominal/Examples" = "HOL-Nominal" +
   750 session "HOL-Nominal-Examples" in "Nominal/Examples" = "HOL-Nominal" +
   752   options [condition = ML_SYSTEM_POLYML, document = false]
   751   options [document = false]
   753   theories
   752   theories
   754     Class3
   753     Class3
   755     CK_Machine
   754     CK_Machine
   756     Compile
   755     Compile
   757     Contexts
   756     Contexts
   836 session "HOL-Mirabelle" in Mirabelle = HOL +
   835 session "HOL-Mirabelle" in Mirabelle = HOL +
   837   options [document = false]
   836   options [document = false]
   838   theories Mirabelle_Test
   837   theories Mirabelle_Test
   839 
   838 
   840 session "HOL-Mirabelle-ex" in "Mirabelle/ex" = "HOL-Mirabelle" +
   839 session "HOL-Mirabelle-ex" in "Mirabelle/ex" = "HOL-Mirabelle" +
   841   options [condition = ML_SYSTEM_POLYML, document = false, timeout = 60]
   840   options [document = false, timeout = 60]
   842   theories Ex
   841   theories Ex
   843 
   842 
   844 session "HOL-Word-SMT_Examples" in SMT_Examples = "HOL-Word" +
   843 session "HOL-Word-SMT_Examples" in SMT_Examples = "HOL-Word" +
   845   options [condition = ML_SYSTEM_POLYML, document = false, quick_and_dirty]
   844   options [document = false, quick_and_dirty]
   846   theories
   845   theories
   847     Boogie
   846     Boogie
   848     SMT_Examples
   847     SMT_Examples
   849     SMT_Word_Examples
   848     SMT_Word_Examples
   850     SMT_Tests
   849     SMT_Tests
   979     Int_Pow
   978     Int_Pow
   980     Lifting_Code_Dt_Test
   979     Lifting_Code_Dt_Test
   981 
   980 
   982 session "HOL-Predicate_Compile_Examples" in Predicate_Compile_Examples = HOL +
   981 session "HOL-Predicate_Compile_Examples" in Predicate_Compile_Examples = HOL +
   983   options [document = false]
   982   options [document = false]
   984   theories [condition = ML_SYSTEM_POLYML]
   983   theories
   985     Examples
   984     Examples
   986     Predicate_Compile_Tests
   985     Predicate_Compile_Tests
   987     Predicate_Compile_Quickcheck_Examples
   986     Predicate_Compile_Quickcheck_Examples
   988     Specialisation_Examples
   987     Specialisation_Examples
   989     IMP_1
   988     IMP_1