aboutsummaryrefslogtreecommitdiffhomepage
path: root/toplevel
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-06-10 21:08:49 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-06-10 21:08:49 +0000
commitc8d73b13c7738d3b24533488e9d31dc6f82daed1 (patch)
tree76dc6a96931bb7395d35f83b92c72e02978833f1 /toplevel
parent412fe23944757811a3522fa7feba73cd0af9fbc0 (diff)
Déplacement de code dans command; MAJ DebugOn
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4119 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'toplevel')
-rw-r--r--toplevel/vernacentries.ml14
1 files changed, 5 insertions, 9 deletions
diff --git a/toplevel/vernacentries.ml b/toplevel/vernacentries.ml
index 33ecab345..8d21c4d76 100644
--- a/toplevel/vernacentries.ml
+++ b/toplevel/vernacentries.ml
@@ -335,8 +335,7 @@ let vernac_definition local id def hook =
| Some r ->
let (evc,env)= Command.get_current_context () in
Some (interp_redexp env evc r) in
- let ref = declare_definition id local bl red_option c typ_opt in
- hook local ref
+ declare_definition id local bl red_option c typ_opt hook
let vernac_start_proof kind sopt (bl,t) lettop hook =
if not(refining ()) then
@@ -362,11 +361,8 @@ let vernac_exact_proof c =
by (Tactics.exact_proof c);
save_named true
-let vernac_assumption (islocal,_ as kind) l =
- List.iter
- (fun (is_coe,(id,c)) ->
- let r = declare_assumption id kind [] c in
- if is_coe then Class.try_add_new_coercion r islocal) l
+let vernac_assumption kind l =
+ List.iter (fun (is_coe,(id,c)) -> declare_assumption id is_coe kind [] c) l
let vernac_inductive f indl = build_mutual indl f
@@ -707,7 +703,7 @@ let vernac_syntactic_definition id c = function
| None -> syntax_definition id c
| Some n ->
let l = list_tabulate (fun _ -> (CHole (dummy_loc),None)) n in
- let c = CApp (dummy_loc,c,l) in
+ let c = CApp (dummy_loc,(false,c),l) in
syntax_definition id c
let vernac_declare_implicits locqid = function
@@ -1054,7 +1050,7 @@ let vernac_check_guard () =
msgnl message
let vernac_debug b =
- set_debug (if b then Tactic_debug.DebugOn else Tactic_debug.DebugOff)
+ set_debug (if b then Tactic_debug.DebugOn 0 else Tactic_debug.DebugOff)
(**************************)