src/HOL/Tools/Predicate_Compile/mode_inference.ML
changeset 55440 721b4561007a
parent 55399 5c8e91f884af
parent 55437 3fd63b92ea3b
child 59481 74f638efffcb
--- a/src/HOL/Tools/Predicate_Compile/mode_inference.ML	Wed Feb 12 10:59:25 2014 +0100
+++ b/src/HOL/Tools/Predicate_Compile/mode_inference.ML	Wed Feb 12 14:32:45 2014 +0100
@@ -71,8 +71,10 @@
 fun mode_of (Context m) = m
   | mode_of (Term m) = m
   | mode_of (Mode_App (d1, d2)) =
-    (case mode_of d1 of Fun (m, m') =>
-        (if eq_mode (m, mode_of d2) then m' else raise Fail "mode_of: derivation has mismatching modes")
+      (case mode_of d1 of
+        Fun (m, m') =>
+          (if eq_mode (m, mode_of d2) then m'
+           else raise Fail "mode_of: derivation has mismatching modes")
       | _ => raise Fail "mode_of: derivation has a non-functional mode")
   | mode_of (Mode_Pair (d1, d2)) =
     Pair (mode_of d1, mode_of d2)
@@ -109,12 +111,12 @@
     (Syntax.string_of_term ctxt (HOLogic.mk_not t)) ^ "(negative premise)"
   | string_of_prem ctxt (Sidecond t) =
     (Syntax.string_of_term ctxt t) ^ "(sidecondition)"
-  | string_of_prem ctxt _ = raise Fail "string_of_prem: unexpected input"
+  | string_of_prem _ _ = raise Fail "string_of_prem: unexpected input"
 
 type mode_analysis_options =
   {use_generators : bool,
-  reorder_premises : bool,
-  infer_pos_and_neg_modes : bool}
+   reorder_premises : bool,
+   infer_pos_and_neg_modes : bool}
 
 (*** check if a type is an equality type (i.e. doesn't contain fun)
   FIXME this is only an approximation ***)
@@ -134,7 +136,7 @@
 
 fun error_of p (_, m) is =
   "  Clauses " ^ commas (map (fn i => string_of_int (i + 1)) is) ^ " of " ^
-        p ^ " violates mode " ^ string_of_mode m
+  p ^ " violates mode " ^ string_of_mode m
 
 fun is_all_input mode =
   let