src/HOL/SMT.thy
changeset 36902 c6bae4456741
parent 36899 bcd6fce5bf06
child 37124 fe22fc54b876
--- a/src/HOL/SMT.thy	Thu May 13 00:44:48 2010 +0200
+++ b/src/HOL/SMT.thy	Wed May 12 22:33:10 2010 -0700
@@ -26,7 +26,7 @@
 
 
 
-section {* Triggers for quantifier instantiation *}
+subsection {* Triggers for quantifier instantiation *}
 
 text {*
 Some SMT solvers support triggers for quantifier instantiation.
@@ -53,7 +53,7 @@
 
 
 
-section {* Higher-order encoding *}
+subsection {* Higher-order encoding *}
 
 text {*
 Application is made explicit for constants occurring with varying
@@ -74,7 +74,7 @@
 
 
 
-section {* First-order logic *}
+subsection {* First-order logic *}
 
 text {*
 Some SMT solvers require a strict separation between formulas and
@@ -91,7 +91,7 @@
 
 
 
-section {* Setup *}
+subsection {* Setup *}
 
 use "Tools/SMT/smt_monomorph.ML"
 use "Tools/SMT/smt_normalize.ML"
@@ -118,7 +118,7 @@
 
 
 
-section {* Configuration *}
+subsection {* Configuration *}
 
 text {*
 The current configuration can be printed by the command
@@ -224,7 +224,7 @@
 
 
 
-section {* Schematic rules for Z3 proof reconstruction *}
+subsection {* Schematic rules for Z3 proof reconstruction *}
 
 text {*
 Several prof rules of Z3 are not very well documented.  There are two