Skip to content

Commit

Permalink
fix(comments) Remove all ddddmmits and scary words from within comments
Browse files Browse the repository at this point in the history
Signed-off-by: jeromesimeon <jeromesimeon@me.com>
  • Loading branch information
jeromesimeon committed Sep 10, 2021
1 parent 36b3640 commit c6d2cf1
Show file tree
Hide file tree
Showing 4 changed files with 1 addition and 52 deletions.
11 changes: 0 additions & 11 deletions compiler/core/CAMP/Typing/TCAMP.v
Original file line number Diff line number Diff line change
Expand Up @@ -225,17 +225,6 @@ Section TCAMP.
inversion H0; subst; rtype_equalizer.
subst. constructor. constructor; eauto.
* discriminate.
(* pgroupBy *)
(*
- inversion tdat; subst.
rtype_equalizer. subst.
induction dl; simpl.
+ left; econstructor; split; eauto. econstructor; eauto.
+ inversion H2; subst.
specialize (IHdl (dtcoll _ _ H4) H4).
destruct (IHp _ _ _ _ _ tenv H1 H3) as [[dout[camp_evaleq tx]]|[s camp_evaleq]].
addddmit.
addddmit. *)
(* passert *)
- destruct (IHp _ _ _ _ _ tenv H1 tdat) as [[dout[camp_evaleq tx]]|camp_evaleq];
rewrite camp_evaleq; simpl; [|eauto].
Expand Down
1 change: 0 additions & 1 deletion compiler/core/Driver/CompCorrectness.v
Original file line number Diff line number Diff line change
Expand Up @@ -1295,7 +1295,6 @@ Section CompCorrectness.
unfold lift_input.
trivial_same_query.
assumption.
a dmit.
Qed.
*)

Expand Down
38 changes: 0 additions & 38 deletions compiler/core/NNRCMR/Optim/NNRCMRRewrite.v
Original file line number Diff line number Diff line change
Expand Up @@ -888,43 +888,6 @@ Section NNRCMRRewrite.
try contradiction; try congruence.
Qed.


(* XXXXXXXXXXXXXXXXXXXXXXXXXXXXXXXX TODO XXXXXXXXXXXXXXXXXXXXXX *)

(* (* KindOfId+M=M *) *)

(* Definition merge_mr_kindofid mr1 mr2 := *)
(* if equiv_decb mr1.(mr_output) mr2.(mr_input) && is_kindofid_mr mr1 then *)
(* let mr := *)
(* mkMR *)
(* mr1.(mr_input) *)
(* mr2.(mr_output) *)
(* mr2.(mr_flat_map) *)
(* mr2.(mr_reduce) *)
(* in *)
(* Some mr *)
(* else *)
(* None. *)

(* Lemma merge_mr_kindofid_correct : *)
(* merge_correct_singleton merge_mr_kindofid. *)
(* Proof. *)
(* unfold merge_correct_singleton. intros m1 m2 m3. *)
(* intros Hdist1 Hdist2. intros. *)
(* unfold merge_mr_kindofid in H0. *)
(* unfold equiv_decb in *. *)
(* dest_eqdec; simpl in *. *)
(* - case_eq (is_kindofid_mr m1); intros; *)
(* rewrite H1 in H0; try congruence. *)
(* unfold mr_chain_eval. *)
(* simpl. *)
(* dest_eqdec; [ | congruence ]. *)
(* a.dmit. *)
(* - discriminate. *)
(* Qed. *)

(* map-id + id-red = map-red *)

(* Java equivalent: MROptimizer.merge_id_reduce_id_dist_map *)
Definition merge_id_reduce_id_dist_map mr1 mr2 :=
if equiv_decb mr1.(mr_output) mr2.(mr_input)
Expand Down Expand Up @@ -1483,4 +1446,3 @@ Section NNRCMRRewrite.
get_mr_chain_vars mrl.(mr_chain).

End NNRCMRRewrite.

3 changes: 1 addition & 2 deletions compiler/core/Updates/UDelta.v
Original file line number Diff line number Diff line change
Expand Up @@ -217,8 +217,7 @@ Section UDelta.
elim (rmap (update Δ₀) l); intros; congruence.
rewrite H.
destruct (rmap (update Δ₀) l); reflexivity.
- addddmit. (* still need work on record update – no easy corresponding query *)
- simpl. addddmit. (* still need work on compose – possibly showing an intermediate lemma that does substitute with AID. *)
(* TODO *)
Qed.
*)

Expand Down

0 comments on commit c6d2cf1

Please sign in to comment.