aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--checker/declarations.ml2
-rw-r--r--kernel/mod_subst.ml2
-rw-r--r--plugins/extraction/haskell.ml2
3 files changed, 3 insertions, 3 deletions
diff --git a/checker/declarations.ml b/checker/declarations.ml
index df8abb256..0e5eb0c23 100644
--- a/checker/declarations.ml
+++ b/checker/declarations.ml
@@ -580,7 +580,7 @@ let update_delta_resolver resolver1 resolver2 =
Equiv (solve_delta_kn resolver2 kn)
in Deltamap.add key new_hint res
| _ -> Deltamap.add key hint res
- with not_found ->
+ with Not_found ->
Deltamap.add key hint res
in
Deltamap.fold apply_res resolver1 empty_delta_resolver
diff --git a/kernel/mod_subst.ml b/kernel/mod_subst.ml
index 8c768b3a5..8b11aa185 100644
--- a/kernel/mod_subst.ml
+++ b/kernel/mod_subst.ml
@@ -643,7 +643,7 @@ let update_delta_resolver resolver1 resolver2 =
Change_equiv_to_inline c ->
Deltamap.add key (Inline (Some c)) res)
| _ -> Deltamap.add key hint res
- with not_found ->
+ with Not_found ->
Deltamap.add key hint res
in
Deltamap.fold apply_res resolver1 empty_delta_resolver
diff --git a/plugins/extraction/haskell.ml b/plugins/extraction/haskell.ml
index 1d698d129..3048db4b7 100644
--- a/plugins/extraction/haskell.ml
+++ b/plugins/extraction/haskell.ml
@@ -295,7 +295,7 @@ let pp_decl = function
try
let ids,s = find_type_custom r in
prlist (fun id -> str (id^" ")) ids ++ str "=" ++ spc () ++ str s
- with not_found ->
+ with Not_found ->
prlist (fun id -> pr_id id ++ str " ") l ++
if t = Taxiom then str "= () -- AXIOM TO BE REALIZED\n"
else str "=" ++ spc () ++ pp_type false l t