Skip to content

Commit

Permalink
Remove some commented Admitted lemmas
Browse files Browse the repository at this point in the history
  • Loading branch information
ymherklotz committed Jan 20, 2024
1 parent edbd370 commit 0a15dc1
Show file tree
Hide file tree
Showing 2 changed files with 0 additions and 55 deletions.
12 changes: 0 additions & 12 deletions src/Compiler.v
Original file line number Diff line number Diff line change
Expand Up @@ -184,18 +184,6 @@ Proof.
- red; intros. subst tp1 tp2. exists p; auto.
Qed.

(* Global Instance TransfIfLink {A: Type} {LA: Linker A} *)
(* (transf: A -> A -> Prop) (TL: TransfLink transf) *)
(* : TransfLink (match_rep transf). *)
(* Admitted. *)

(* Lemma total_rep_match: *)
(* forall (A B: Type) (n: list B) (f: A -> B -> A) *)
(* (rel: A -> A -> Prop) (prog: A), *)
(* (forall b p, rel p (f p b)) -> *)
(* match_rep rel prog (fold_left f n prog). *)
(* Proof. Admitted. *)

Lemma total_if_match:
forall (A: Type) (flag: unit -> bool) (f: A -> A)
(rel: A -> A -> Prop) (prog: A),
Expand Down
43 changes: 0 additions & 43 deletions src/hls/DHTLgenproof.v
Original file line number Diff line number Diff line change
Expand Up @@ -2364,49 +2364,6 @@ Proof.
eapply PTree.elements_correct; eauto.
Qed.

(* Lemma lt_max_resources_in_block : *)
(* forall bb a pc x x0, *)
(* In x (concat bb) -> *)
(* In x0 (pred_uses x) -> *)
(* Ple x0 (max_pred_block a pc bb). *)
(* Proof. *)
(* induction bb. *)
(* - intros. cbn in *. inv H. *)
(* - intros. cbn in *. *)

(* Lemma lt_max_resources_lt_a : *)
(* forall bb x x0 a k v, *)
(* In x (concat bb) -> *)
(* In x0 (pred_uses x) -> *)
(* Ple x0 a -> *)
(* Ple x0 (max_pred_block a k v). *)
(* Proof. Admitted. *)

(* Definition inductive_p final fld := *)
(* forall pc bb, *)
(* final ! pc = Some bb -> *)
(* Forall (fun i0 : instr => Forall (fun x2 : positive => Ple x2 fld) (pred_uses i0)) (concat bb). *)

(* Lemma lt_max_resource_predicate_Forall : *)
(* forall f pc bb, *)
(* f.(GibleSubPar.fn_code) ! pc = Some bb -> *)
(* Forall (fun i0 : instr => Forall (fun x2 : positive => Ple x2 (max_pred_function f)) (pred_uses i0)) (concat bb). *)
(* Proof. *)
(* unfold max_pred_function. *)
(* intro f. *)
(* match goal with |- ?g => replace g with (inductive_p (fn_code f) (PTree.fold max_pred_block (fn_code f) 1%positive)) by auto end. *)
(* eapply PTree_Properties.fold_rec; unfold inductive_p; intros; cbn in *. *)
(* - eapply H0. erewrite H. eauto. *)
(* - now rewrite PTree.gempty in H. *)
(* - destruct (peq k pc); subst. *)
(* + rewrite PTree.gss in H2. inv H2. *)
(* eapply Forall_forall; intros. eapply Forall_forall; intros. eauto using lt_max_resources_in_block. *)
(* + rewrite PTree.gso in H2 by auto. *)
(* eapply H1 in H2. eapply Forall_forall; intros. eapply Forall_forall; intros. *)
(* eapply Forall_forall in H2; eauto. eapply Forall_forall in H2; eauto. *)
(* eauto using lt_max_resources_lt_a. *)
(* Qed. *)

Lemma lt_max_resource_predicate_Forall :
forall f pc bb,
f.(GibleSubPar.fn_code) ! pc = Some bb ->
Expand Down

0 comments on commit 0a15dc1

Please sign in to comment.