src/HOL/ROOT
changeset 51558 91f8bed6d0a4
parent 51553 63327f679cff
child 51559 320907e48a9e
--- a/src/HOL/ROOT	Wed Mar 27 17:58:07 2013 +0100
+++ b/src/HOL/ROOT	Wed Mar 27 18:04:21 2013 +0100
@@ -16,7 +16,7 @@
   description {*
     HOL-Main with explicit proof terms.
   *}
-  options [document = false, proofs = 2]
+  options [document = false, proofs = 2, skip_proofs = false]
   theories Main
   files
     "Tools/Quickcheck/Narrowing_Engine.hs"
@@ -354,14 +354,14 @@
   theories Decision_Procs
 
 session "HOL-Proofs-ex" in "Proofs/ex" = "HOL-Proofs" +
-  options [document = false, proofs = 2, parallel_proofs = 0]
+  options [document = false, proofs = 2, skip_proofs = false, parallel_proofs = 0]
   theories Hilbert_Classical
 
 session "HOL-Proofs-Extraction" in "Proofs/Extraction" = "HOL-Proofs" +
   description {*
     Examples for program extraction in Higher-Order Logic.
   *}
-  options [condition = ISABELLE_POLYML, proofs = 2, parallel_proofs = 0]
+  options [condition = ISABELLE_POLYML, proofs = 2, skip_proofs = false, parallel_proofs = 0]
   theories [document = false]
     "~~/src/HOL/Library/Code_Target_Numeral"
     "~~/src/HOL/Library/Monad_Syntax"
@@ -386,7 +386,8 @@
     The paper "More Church-Rosser Proofs (in Isabelle/HOL)" describes the whole
     theory (see http://www.in.tum.de/~nipkow/pubs/jar2001.html).
   *}
-  options [document_graph, print_mode = "no_brackets", proofs = 2, parallel_proofs = 0]
+  options [document_graph, print_mode = "no_brackets", proofs = 2, skip_proofs = false,
+    parallel_proofs = 0]
   theories [document = false]
     "~~/src/HOL/Library/Code_Target_Int"
   theories
@@ -535,7 +536,6 @@
     Tarski
     Classical
     Set_Theory
-    Meson_Test
     Termination
     Coherent
     PresburgerEx
@@ -561,6 +561,8 @@
     Parallel_Example
     IArray_Examples
   theories SVC_Oracle
+  theories [skip_proofs = false]
+    Meson_Test
   theories [condition = SVC_HOME]
     svc_test
   theories [condition = ZCHAFF_HOME]
@@ -742,7 +744,8 @@
   theories WordExamples
 
 session "HOL-Statespace" in Statespace = HOL +
-  theories StateSpaceEx
+  theories [skip_proofs = false]
+    StateSpaceEx
   files "document/root.tex"
 
 session "HOL-NSA" in NSA = HOL +