src/HOL/Tools/SMT2/smt2_config.ML
changeset 57229 489083abce44
parent 57209 7ffa0f7e2775
child 57230 ec5ff6bb2a92
--- a/src/HOL/Tools/SMT2/smt2_config.ML	Thu Jun 12 01:00:49 2014 +0200
+++ b/src/HOL/Tools/SMT2/smt2_config.ML	Thu Jun 12 01:00:49 2014 +0200
@@ -47,7 +47,7 @@
 
   (*setup*)
   val print_setup: Proof.context -> unit
-end
+end;
 
 structure SMT2_Config: SMT2_CONFIG =
 struct
@@ -246,4 +246,4 @@
     \and the values of SMT configuration options"
     (Scan.succeed (Toplevel.keep (print_setup o Toplevel.context_of)))
 
-end
+end;