aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel
diff options
context:
space:
mode:
authorGravatar courtieu <courtieu@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-12-16 14:34:13 +0000
committerGravatar courtieu <courtieu@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-12-16 14:34:13 +0000
commit80ef72aa037175549f396e9618274ba69a81cf80 (patch)
treef2b1c3e66f58c552eeac83e67216a89a96b56bff /toplevel
parentb076264235980e60d51a5d0b8d3a4e9c3f4d82eb (diff)
Moving bullets (-, +, *) into stand-alone commands instead of being
part of a tactic. WARNING: Coqide needs to be adapted. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14794 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'toplevel')
-rw-r--r--toplevel/ide_slave.ml1
-rw-r--r--toplevel/vernacentries.ml15
-rw-r--r--toplevel/vernacexpr.ml3
3 files changed, 15 insertions, 4 deletions
diff --git a/toplevel/ide_slave.ml b/toplevel/ide_slave.ml
index 31a651279..42ecb75bc 100644
--- a/toplevel/ide_slave.ml
+++ b/toplevel/ide_slave.ml
@@ -208,6 +208,7 @@ let rec attribute_of_vernac_command = function
| VernacProof _ -> []
| VernacProofMode _ -> []
+ | VernacBullet _ -> [SolveCommand]
| VernacSubproof _ -> [SolveCommand]
| VernacEndSubproof -> [SolveCommand]
diff --git a/toplevel/vernacentries.ml b/toplevel/vernacentries.ml
index 435d85233..a04b167cb 100644
--- a/toplevel/vernacentries.ml
+++ b/toplevel/vernacentries.ml
@@ -645,12 +645,11 @@ let command_focus = Proof.new_focus_kind ()
let focus_command_cond = Proof.no_cond command_focus
-let vernac_solve n bullet tcom b =
+let vernac_solve n tcom b =
if not (refining ()) then
error "Unknown command of the non proof-editing mode.";
let p = Proof_global.give_me_the_proof () in
Proof.transaction p begin fun () ->
- Option.iter (Proof_global.Bullet.put p) bullet ;
solve_nth n (Tacinterp.hide_interp tcom None) ~with_end_tac:b;
(* in case a strict subtree was completed,
go back to the top of the prooftree *)
@@ -1367,6 +1366,15 @@ let vernac_end_subproof () =
let p = Proof_global.give_me_the_proof () in
Proof.unfocus subproof_kind p ; print_subgoals ()
+
+let vernac_bullet (bullet:Proof_global.Bullet.t) =
+ let p = Proof_global.give_me_the_proof () in
+ Proof.transaction p
+ (fun () -> Proof_global.Bullet.put p bullet);
+ (* Makes the focus visible in emacs by re-printing the goal. *)
+ if !Flags.print_emacs then print_subgoals ();;
+
+
let vernac_show = function
| ShowGoal goalref ->
if !pcoq <> None then (Option.get !pcoq).show_goal goalref
@@ -1459,7 +1467,7 @@ let interp c = match c with
| VernacDeclareClass id -> vernac_declare_class id
(* Solving *)
- | VernacSolve (n,bullet,tac,b) -> vernac_solve n bullet tac b
+ | VernacSolve (n,tac,b) -> vernac_solve n tac b
| VernacSolveExistential (n,c) -> vernac_solve_existential n c
(* Auxiliary file and library management *)
@@ -1519,6 +1527,7 @@ let interp c = match c with
| VernacBacktrack (snum,pnum,naborts) -> vernac_backtrack snum pnum naborts
| VernacFocus n -> vernac_focus n
| VernacUnfocus -> vernac_unfocus ()
+ | VernacBullet b -> vernac_bullet b
| VernacSubproof n -> vernac_subproof n
| VernacEndSubproof -> vernac_end_subproof ()
| VernacShow s -> vernac_show s
diff --git a/toplevel/vernacexpr.ml b/toplevel/vernacexpr.ml
index b1ab3bdce..f2e2c0ac7 100644
--- a/toplevel/vernacexpr.ml
+++ b/toplevel/vernacexpr.ml
@@ -284,7 +284,7 @@ type vernac_expr =
(* Solving *)
- | VernacSolve of int * bullet option * raw_tactic_expr * bool
+ | VernacSolve of int * raw_tactic_expr * bool
| VernacSolveExistential of int * constr_expr
(* Auxiliary file and library management *)
@@ -353,6 +353,7 @@ type vernac_expr =
| VernacBacktrack of int*int*int
| VernacFocus of int option
| VernacUnfocus
+ | VernacBullet of bullet
| VernacSubproof of int option
| VernacEndSubproof
| VernacShow of showable