diff -r 9537bf1c4853 -r 5b7a9633cfa8 src/HOL/SMT.thy --- a/src/HOL/SMT.thy Sun Nov 02 18:21:14 2014 +0100 +++ b/src/HOL/SMT.thy Sun Nov 02 18:21:45 2014 +0100 @@ -2,7 +2,7 @@ Author: Sascha Boehme, TU Muenchen *) -header {* Bindings to Satisfiability Modulo Theories (SMT) solvers based on SMT-LIB 2 *} +section {* Bindings to Satisfiability Modulo Theories (SMT) solvers based on SMT-LIB 2 *} theory SMT imports Divides