aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel/vernacentries.ml
diff options
context:
space:
mode:
Diffstat (limited to 'toplevel/vernacentries.ml')
-rw-r--r--toplevel/vernacentries.ml6
1 files changed, 3 insertions, 3 deletions
diff --git a/toplevel/vernacentries.ml b/toplevel/vernacentries.ml
index 42c36f519..71f7f39a3 100644
--- a/toplevel/vernacentries.ml
+++ b/toplevel/vernacentries.ml
@@ -259,7 +259,7 @@ let print_namespace ns =
begin match match_dirpath ns dir with
| Some [] as y -> y
| Some (a::ns') ->
- if Names.id_ord a id = 0 then Some ns'
+ if Int.equal (Names.id_ord a id) 0 then Some ns'
else None
| None -> None
end
@@ -272,7 +272,7 @@ let print_namespace ns =
begin match match_modulepath ns mp with
| Some [] as y -> y
| Some (a::ns') ->
- if Names.id_ord a id = 0 then Some ns'
+ if Int.equal (Names.id_ord a id) 0 then Some ns'
else None
| None -> None
end
@@ -1551,7 +1551,7 @@ let vernac_undoto n =
let vernac_focus gln =
let p = Proof_global.give_me_the_proof () in
let n = match gln with None -> 1 | Some n -> n in
- if n = 0 then
+ if Int.equal n 0 then
Errors.error "Invalid goal number: 0. Goal numbering starts with 1."
else
Proof.focus focus_command_cond () n p; print_subgoals ()