Skip to content

Commit dace0dd

Browse files
committed
Use ocp-indent and reindent
1 parent 60707f6 commit dace0dd

File tree

6 files changed

+371
-369
lines changed

6 files changed

+371
-369
lines changed

.ocp-indent

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -0,0 +1,2 @@
1+
JaneStreet
2+
match_clause = 4

src/mtac2Interp.ml

Lines changed: 8 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -11,13 +11,13 @@ let get_its_info gls = Mtac2ProofInfos.get_info gls.Evd.sigma gls.it
1111
(** *)
1212
let tcl_change_info_gen info_gen =
1313
(fun gls ->
14-
let it = Evd.sig_it gls in
15-
let concl = Tacmach.pf_concl gls in
16-
let hyps = Goal.V82.hyps (Tacmach.project gls) it in
17-
let extra = Goal.V82.extra (Tacmach.project gls) it in
18-
let (gl,ev,sigma) = Goal.V82.mk_goal (Tacmach.project gls) hyps concl (info_gen extra) in
19-
let sigma = Goal.V82.partial_solution sigma it ev in
20-
{it = [gl] ; sigma= sigma; } )
14+
let it = Evd.sig_it gls in
15+
let concl = Tacmach.pf_concl gls in
16+
let hyps = Goal.V82.hyps (Tacmach.project gls) it in
17+
let extra = Goal.V82.extra (Tacmach.project gls) it in
18+
let (gl,ev,sigma) = Goal.V82.mk_goal (Tacmach.project gls) hyps concl (info_gen extra) in
19+
let sigma = Goal.V82.partial_solution sigma it ev in
20+
{it = [gl] ; sigma= sigma; } )
2121

2222
(** Updates the info of the evar maps *)
2323
let tcl_change_info info gls =
@@ -56,7 +56,7 @@ let interp_mproof_command () =
5656
(** Interpreter of a mtactic *)
5757
let interp_instr instr =
5858
match instr with
59-
| Mtac2Instr.Mtac2_constr c -> Mtac2Run.run_tac c
59+
| Mtac2Instr.Mtac2_constr c -> Mtac2Run.run_tac c
6060

6161
(** Interpreter of a constr :
6262
- Interpretes the constr

src/mtac2ProofInfos.ml

Lines changed: 12 additions & 13 deletions
Original file line numberDiff line numberDiff line change
@@ -1,12 +1,11 @@
11
(**
2-
This module concerns the state of the proof tree
2+
This module concerns the state of the proof tree
33
*)
44

55
(** *)
66
type split_tree=
77
Skip_patt of Names.Id.Set.t * split_tree
8-
| Split_patt of Names.Id.Set.t * Names.inductive *
9-
(bool array * (Names.Id.Set.t * split_tree) option) array
8+
| Split_patt of Names.Id.Set.t * Names.inductive * (bool array * (Names.Id.Set.t * split_tree) option) array
109
| Close_patt of split_tree
1110
| End_patt of (Names.Id.t * (int * int))
1211

@@ -19,14 +18,14 @@ type elim_kind =
1918
type recpath = int option*Declarations.wf_paths
2019

2120
type per_info =
22-
{per_casee:Term.constr;
23-
per_ctype:Term.types;
24-
per_ind:Names.inductive;
25-
per_pred:Term.constr;
26-
per_args:Term.constr list;
27-
per_params:Term.constr list;
28-
per_nparams:int;
29-
per_wf:recpath}
21+
{per_casee:Term.constr;
22+
per_ctype:Term.types;
23+
per_ind:Names.inductive;
24+
per_pred:Term.constr;
25+
per_args:Term.constr list;
26+
per_params:Term.constr list;
27+
per_nparams:int;
28+
per_wf:recpath}
3029

3130
type elim_type =
3231
ET_Case_analysis
@@ -39,7 +38,7 @@ type stack_info =
3938
| Focus_claim
4039

4140
type pm_info =
42-
{ pm_stack : stack_info list}
41+
{ pm_stack : stack_info list}
4342

4443
(** Create a new field in datatype used to store additional information in evar maps*)
4544
let info = Evd.Store.field ()
@@ -61,7 +60,7 @@ let proof_cond = Proof.no_cond proof_focus
6160
(** focus on the proof *)
6261
let focus p =
6362
let inf = get_stack p in
64-
Printf.printf "____focus\n%!";
63+
Printf.printf "____focus\n%!";
6564
Proof_global.simple_with_current_proof
6665
(fun _ -> Proof.focus proof_cond inf 1)
6766

src/mtac2Run.ml

Lines changed: 5 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -28,9 +28,9 @@ let run_tac t =
2828
let (sigma, t) = pretypeT env sigma concl c in
2929
let r = run (env, sigma) c in
3030
match r with
31-
| Val (sigma', _, v) ->
32-
(Proofview.Unsafe.tclEVARS sigma')
33-
<*> (Proofview.Refine.refine ~unsafe:false (fun s->(s, v)))
34-
| Err (_, _, e) ->
35-
Errors.error ("Uncaught exception: " ^ (Pp.string_of_ppcmds (Termops.print_constr e)))
31+
| Val (sigma', _, v) ->
32+
(Proofview.Unsafe.tclEVARS sigma')
33+
<*> (Proofview.Refine.refine ~unsafe:false (fun s->(s, v)))
34+
| Err (_, _, e) ->
35+
Errors.error ("Uncaught exception: " ^ (Pp.string_of_ppcmds (Termops.print_constr e)))
3636
end

0 commit comments

Comments
 (0)