aboutsummaryrefslogtreecommitdiff
path: root/tactics/contradiction.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 /tactics/contradiction.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 'tactics/contradiction.ml')
-rw-r--r--tactics/contradiction.ml16
1 files changed, 8 insertions, 8 deletions
diff --git a/tactics/contradiction.ml b/tactics/contradiction.ml
index 56e8e7a11f..1f5a6380fd 100644
--- a/tactics/contradiction.ml
+++ b/tactics/contradiction.ml
@@ -66,10 +66,10 @@ let contradiction_context =
| d :: rest ->
let id = NamedDecl.get_id d in
let typ = nf_evar sigma (NamedDecl.get_type d) in
- let typ = whd_all env sigma typ in
+ let typ = whd_all env sigma typ in
if is_empty_type env sigma typ then
- simplest_elim (mkVar id)
- else match EConstr.kind sigma typ with
+ simplest_elim (mkVar id)
+ else match EConstr.kind sigma typ with
| Prod (na,t,u) when is_empty_type env sigma u ->
let is_unit_or_eq = match_with_unit_or_eq_type env sigma t in
Tacticals.New.tclORELSE
@@ -84,17 +84,17 @@ let contradiction_context =
simplest_elim (mkApp (mkVar id,[|p|]))
| None ->
Tacticals.New.tclZEROMSG (Pp.str"Not a negated unit type."))
- (Proofview.tclORELSE
+ (Proofview.tclORELSE
(Proofview.Goal.enter begin fun gl ->
let is_conv_leq = Tacmach.New.pf_apply is_conv_leq gl in
- filter_hyp (fun typ -> is_conv_leq typ t)
- (fun id' -> simplest_elim (mkApp (mkVar id,[|mkVar id'|])))
+ filter_hyp (fun typ -> is_conv_leq typ t)
+ (fun id' -> simplest_elim (mkApp (mkVar id,[|mkVar id'|])))
end)
begin function (e, info) -> match e with
- | Not_found -> seek_neg rest
+ | Not_found -> seek_neg rest
| e -> Proofview.tclZERO ~info e
end)
- | _ -> seek_neg rest
+ | _ -> seek_neg rest
in
let hyps = Proofview.Goal.hyps gl in
seek_neg hyps