src/HOL/Analysis/metric_arith.ML
changeset 74546 6df92c387063
parent 74545 6c123914883a
child 74547 54055f568d76
--- a/src/HOL/Analysis/metric_arith.ML	Tue Oct 19 14:58:22 2021 +0200
+++ b/src/HOL/Analysis/metric_arith.ML	Tue Oct 19 15:03:00 2021 +0200
@@ -1,9 +1,17 @@
-signature METRIC_ARITH = sig
+(*  Title:      HOL/Analysis/metric_arith.ML
+    Author:     Maximilian Schäffeler (port from HOL Light)
+
+A decision procedure for metric spaces.
+*)
+
+signature METRIC_ARITH =
+sig
+  val trace: bool Config.T
   val metric_arith_tac : Proof.context -> int -> tactic
-  val trace: bool Config.T
 end
 
-structure MetricArith : METRIC_ARITH = struct
+structure Metric_Arith : METRIC_ARITH =
+struct
 
 fun default d x = case x of SOME y => SOME y | NONE => d
 
@@ -318,4 +326,5 @@
   IF_UNSOLVED' (SUBPROOF (fn {context=ctxt', ...} =>
     trace_tac ctxt' "Focused on subgoal" THEN
     elim_exists ctxt') ctxt)
+
 end