aboutsummaryrefslogtreecommitdiff
path: root/engine/proofview.ml
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2019-11-21 15:38:39 +0100
committerEmilio Jesus Gallego Arias2019-11-21 15:38:39 +0100
commitd016f69818b30b75d186fb14f440b93b0518fc66 (patch)
tree32cd948273f79a2c01ad27b4ed0244ea60d7e2f9 /engine/proofview.ml
parentb680b06b31c27751a7d551d95839aea38f7fbea1 (diff)
[coq] Untabify the whole ML codebase.
We also remove trailing whitespace. Script used: ```bash for i in `find . -name '*.ml' -or -name '*.mli' -or -name '*.mlg'`; do expand -i "$i" | sponge "$i"; sed -e's/[[:space:]]*$//' -i.bak "$i"; done ```
Diffstat (limited to 'engine/proofview.ml')
-rw-r--r--engine/proofview.ml14
1 files changed, 7 insertions, 7 deletions
diff --git a/engine/proofview.ml b/engine/proofview.ml
index d6f5aab1d1..ed44372045 100644
--- a/engine/proofview.ml
+++ b/engine/proofview.ml
@@ -130,7 +130,7 @@ let focus_context (left,right) =
i]. *)
let focus_sublist i j l =
let (left,sub_right) = CList.goto (i-1) l in
- let (sub, right) =
+ let (sub, right) =
try CList.chop (j-i+1) sub_right
with Failure _ -> raise CList.IndexOutOfRange
in
@@ -479,7 +479,7 @@ let fold_left2_goal i s l =
let err =
return () >>= fun () -> (* Delay the computation of list lengths. *)
tclZERO (SizeMismatch (CList.length initial.comb,CList.length l))
- in
+ in
Proof.List.fold_left2 err begin fun ((r,subgoals) as cur) goal a ->
Solution.get >>= fun step ->
match cleared_alias step goal with
@@ -515,7 +515,7 @@ let fold_left2_goal i s l =
let tclDISPATCHGEN0 join tacs =
match tacs with
| [] ->
- begin
+ begin
let open Proof in
Comb.get >>= function
| [] -> tclUNIT (join [])
@@ -1012,7 +1012,7 @@ module Unsafe = struct
let tclEVARSADVANCE evd =
Pv.modify (fun ps -> { ps with solution = evd; comb = undefined evd ps.comb })
- let tclEVARUNIVCONTEXT ctx =
+ let tclEVARUNIVCONTEXT ctx =
Pv.modify (fun ps -> { ps with solution = Evd.set_universe_context ps.solution ctx })
let reset_future_goals p =
@@ -1229,7 +1229,7 @@ module V82 = struct
let (_goals,evd) = Evd.Monad.List.map map comb ps.solution in
{ ps with solution = evd; }
end
-
+
let has_unresolved_evar pv =
Evd.has_undefined pv.solution
@@ -1238,8 +1238,8 @@ module V82 = struct
let undef = Evd.undefined_map pv.solution in
let goals = CList.rev_map fst (Evar.Map.bindings undef) in
{ pv with comb = List.map with_empty_state goals }
-
-
+
+
let top_goals initial { solution=solution; } =
let goals = CList.map (fun (t,_) -> fst (Constr.destEvar (EConstr.Unsafe.to_constr t))) initial in