Skip to content

Commit c23b71a

Browse files
Jesse Michael Hanfpvandoorn
Jesse Michael Han
authored andcommitted
Anonymize TODOs and floris_mixture
1 parent e804a71 commit c23b71a

File tree

9 files changed

+31
-31
lines changed

9 files changed

+31
-31
lines changed

src/abstract_forcing.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -57,7 +57,7 @@ instance : forcing_notion punit := order_top.mk (by finish)
5757

5858
instance forcing_notion_complete_boolean_algebra {α : Type u} [complete_boolean_algebra α] : forcing_notion α := order_top.mk (by finish)
5959

60-
--TODO(jesse) rewrite in terms of pSet.rec and Name.rec
60+
--TODO() rewrite in terms of pSet.rec and Name.rec
6161
def pSet_equiv_trivial_name : pSet.{u} ≃ (punit-name : Type (u+1)) :=
6262
{ to_fun := λ u,
6363
begin

src/bfol.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -804,7 +804,7 @@ by { ext, simp [bd_not] }
804804
(s : bounded_term L n) : (f ⊓ g)[s/0] = (f[s/0] ⊓ g[s/0]) :=
805805
by { ext, simp[bd_and, bd_not] }
806806

807-
-- --TODO(floris)
807+
-- --TODO()
808808
-- lemma realize_subst_bt {L : Language} {S : bStructure L β} : ∀{n n' l}
809809
-- (t : bounded_preterm L (n+n'+1) l)
810810
-- (s : bounded_term L n') (v : dvector S n) (v' : dvector S n') (v'' : dvector S l),

src/bvm.lean

Lines changed: 12 additions & 12 deletions
Original file line numberDiff line numberDiff line change
@@ -57,7 +57,7 @@ by {rw[inf_comm], apply bv_cases_left, simpa only [inf_comm]}
5757
lemma bv_specialize {ι : Type*} {s : ι → 𝔹} (i : ι) {b : 𝔹} {h : s i ≤ b} :
5858
(⨅(i:ι), s i) ≤ b := infi_le_of_le i h
5959

60-
--TODO(jesse) write the version of this for an arbitrary list of instantiations
60+
--TODO() write the version of this for an arbitrary list of instantiations
6161
lemma bv_specialize_twice {ι : Type*} {s : ι → 𝔹} (i j : ι) {b : 𝔹} {h : s i ⊓ s j ≤ b} :
6262
(⨅(i:ι), s i) ≤ b :=
6363
begin
@@ -589,7 +589,7 @@ poset_yoneda_inv Γ subset_trans $ le_inf ‹_› ‹_›
589589
-- apply subset_trans
590590
-- end
591591

592-
-- TODO(jesse): mark this as simp
592+
-- TODO(): mark this as simp
593593
lemma mem_of_mem_subset {x y z : bSet 𝔹} {Γ} (H₂ : Γ ≤ y ⊆ᴮ z) (H₁ : Γ ≤ x ∈ᴮ y) : Γ ≤ x ∈ᴮ z :=
594594
by {rw[subset_unfold'] at H₂, from H₂ x ‹_›}
595595

@@ -636,7 +636,7 @@ begin
636636
from (poset_yoneda_inv _ (h_congr _ _) this)
637637
end
638638

639-
-- TODO(jesse) maybe replace this with typeclasses instead?
639+
-- TODO() maybe replace this with typeclasses instead?
640640
@[reducible]def B_ext (ϕ : bSet 𝔹 → 𝔹) : Prop :=
641641
∀ x y, x =ᴮ y ⊓ ϕ x ≤ ϕ y
642642

@@ -734,7 +734,7 @@ lemma bv_cc.mk_iff {Γ} {x y : bSet 𝔹} : Γ ≤ x =ᴮ y ↔ (@quotient.mk _
734734

735735
lemma bv_cc.mk {Γ} {x y : bSet 𝔹} (H : Γ ≤ x =ᴮ y) : (@quotient.mk _ (b_setoid Γ) x) = (@quotient.mk _ (b_setoid Γ) y) := bv_cc.mk_iff.mp ‹_›
736736

737-
-- TODO(jesse): automate the generation of these lemmas with typeclasses
737+
-- TODO(): automate the generation of these lemmas with typeclasses
738738
def b_setoid_mem (Γ : 𝔹) : quotient (b_setoid Γ) → quotient (b_setoid Γ) → Prop :=
739739
@quotient.lift₂ (bSet 𝔹) (bSet 𝔹) Prop (b_setoid Γ) (b_setoid Γ) (λ x y, Γ ≤ x ∈ᴮ y)
740740
begin
@@ -948,7 +948,7 @@ begin
948948
apply bv_or_elim; [apply bv_use (ulift.up ff), apply bv_use (ulift.up tt)]; refl
949949
end
950950

951-
def floris_mixture {ι : Type u} (a : ι → 𝔹) (u : ι → bSet 𝔹) : bSet 𝔹 :=
951+
def anon_mixture {ι : Type u} (a : ι → 𝔹) (u : ι → bSet 𝔹) : bSet 𝔹 :=
952952
⟨Σ(i : ι), (u i).type, λx, (u x.fst).func x.snd, λx, a x.fst ⊓ (u x.fst).bval x.snd⟩
953953

954954
/-- Mixing lemma, c.f. Bell's book or Lemma 1 of Hamkins-Seabold -/
@@ -980,7 +980,7 @@ begin
980980
split; [specialize this (ulift.up ff), specialize this (ulift.up tt)]; exact this
981981
end
982982

983-
-- TODO(jesse) try proving mixing_lemma with floris_mixture and see if anything goes wrong
983+
-- TODO() try proving mixing_lemma with _mixture and see if anything goes wrong
984984

985985
/-- In particular, the mixing lemma applies when the weights (a_i) form an antichain and the indexing is injective -/
986986
lemma h_star_of_antichain_injective {ι : Type u} {a : ι → 𝔹} {τ : ι → bSet 𝔹} {h_anti : antichain (a '' set.univ)} {h_inj : function.injective a} :
@@ -1549,7 +1549,7 @@ by {apply top_unique, rw[<-H_top], apply mem.mk'}
15491549
by simp
15501550

15511551
/--
1552-
TODO(jesse): this name should really belong to check_mem instead
1552+
TODO(): this name should really belong to check_mem instead
15531553
-/
15541554
@[simp]lemma mem_check_of_mem {x : pSet} {i : x.type} {Γ : 𝔹} : Γ ≤ ((x.func i) ̌) ∈ᴮ (x̌) :=
15551555
begin
@@ -1676,7 +1676,7 @@ begin
16761676
rw[this] at H, conv{to_rhs, rw[<-H]}, simp }
16771677
end
16781678

1679-
-- TODO(jesse): refactor this so that the conclusion is simply Γ ≤ ¬ (x̌ ∈ᴮ y̌)
1679+
-- TODO(): refactor this so that the conclusion is simply Γ ≤ ¬ (x̌ ∈ᴮ y̌)
16801680
lemma check_not_mem {x y : pSet} : x ∉ y → ∀ {Γ : 𝔹}, Γ ≤ x̌ ∈ᴮ y̌ → Γ ≤ ⊥ :=
16811681
by {intro H, replace H := not_check_mem_iff.mp H, intros Γ HΓ, rwa ←H}
16821682

@@ -1731,7 +1731,7 @@ end
17311731
@[simp]lemma check_exists_mem {y : pSet} (H_exists_mem : ∃ z, z ∈ y ) {Γ : 𝔹} : Γ ≤ exists_mem y̌ :=
17321732
by { rcases H_exists_mem with ⟨z,Hz⟩, apply bv_use ž, simp* }
17331733

1734-
-- note(jesse): this lemma is not true; one also requires that x is a check-name
1734+
-- note(): this lemma is not true; one also requires that x is a check-name
17351735
-- lemma definite_mem_definite_iff_of_subset_check {x y : bSet 𝔹} (H_definite₁ : is_definite x) (H_definite₂ : is_definite y) (H_sub : ∃ z : pSet, ⊤ ≤ y ⊆ᴮ ž) : ⊤ ≤ x ∈ᴮ y ↔ ∃ j : y.type, ⊤ ≤ x =ᴮ y.func j :=
17361736
-- begin
17371737
-- refine ⟨_,_⟩; intro H,
@@ -1842,7 +1842,7 @@ end
18421842

18431843
lemma collect_spec₂ {Γ : 𝔹} (H_AE : Γ ≤ ⨅ i : u.type, u.bval i ⟹ ⨆ w, ϕ (u.func i) w) :
18441844
Γ ≤ ⨅ w, w ∈ᴮ collect ϕ h_congr_right h_congr_left u ⟹ ⨆ z, z ∈ᴮ u ⊓ ϕ z w :=
1845-
begin -- TODO(jesse): prove mem_collect_iff
1845+
begin -- TODO(): prove mem_collect_iff
18461846
bv_intro w, bv_imp_intro Hw_mem, rw mem_unfold at Hw_mem, bv_cases_at Hw_mem i Hi,
18471847
apply bv_use (u.func i), bv_split, apply bv_rw' Hi_right,
18481848
{ refine B_ext_inf _ _,
@@ -2016,7 +2016,7 @@ prefix `𝒫`:80 := bv_powerset
20162016
-- def bv_powerset' (u : bSet 𝔹) : bSet 𝔹 :=
20172017
-- ⟨u.type → 𝔹, λ f, set_of_indicator' f, λ f, ⊤⟩
20182018

2019-
--TODO (jesse) try proving bv_powerset and bv_powerset' are equivalent
2019+
--TODO () try proving bv_powerset and bv_powerset' are equivalent
20202020

20212021
-- example {u : bSet 𝔹} : bv_powerset u =ᴮ bv_powerset' u = ⊤ :=
20222022
-- begin
@@ -2295,7 +2295,7 @@ begin
22952295
change _ ≤ bSet.insert1 0 0 =ᴮ bSet.insert1 0 ∅,
22962296
convert bv_refl, unfold has_zero.zero, unfold of_nat, unfold pSet.of_nat, rw check_empty_eq_empty
22972297
end
2298-
--TODO(jesse): add simp lemmas ensuing (0 : bSet 𝔹) is the simp normal form of (∅̌), (of_nat 0), etc
2298+
--TODO(): add simp lemmas ensuing (0 : bSet 𝔹) is the simp normal form of (∅̌), (of_nat 0), etc
22992299

23002300
lemma forall_empty {Γ : 𝔹} {ϕ : bSet 𝔹 → 𝔹} : Γ ≤ ⨅ x, x ∈ᴮ ∅ ⟹ ϕ x :=
23012301
begin

src/bvm_extras.lean

Lines changed: 6 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -1720,7 +1720,7 @@ begin
17201720
bv_cases_at H_right' s, apply bv_use s, bv_split, refine le_inf _ ‹_›,
17211721
refine le_inf (le_inf _ _) ‹_›,
17221722
{apply bv_rw' (bv_symm ‹_ ≤ g =ᴮ func (𝒫 prod x y) s›), simp, from ‹_›},
1723-
-- TODO(jesse) why does apply fail to generate a motive for bv_rw'?
1723+
-- TODO() why does apply fail to generate a motive for bv_rw'?
17241724
bv_intro w₁, bv_imp_intro Hw₁, replace H_left_right := H_left_right w₁ ‹_›,
17251725
bv_cases_at H_left_right w₂, apply bv_use w₂, bv_split, refine le_inf ‹_› _,
17261726
apply bv_rw' (bv_symm ‹_ ≤ g =ᴮ func (𝒫 prod x y) s›), simp, from ‹_› }
@@ -1763,8 +1763,8 @@ begin
17631763
bv_split_at H, rw[mem_unfold] at H_left H_right,
17641764
bv_cases_at H_left pr₁ Hpr₁, bv_cases_at H_right pr₂ Hpr₂,
17651765
cases pr₁ with i j, cases pr₂ with i' j', simp at *, repeat{auto_cases},
1766-
rw[pair_eq_pair_iff] at Hpr₁_right Hpr₂_right, auto_cases, -- floris, don't look at the tactic state
1767-
have := @H_ext i i' Γ_4 (by bv_cc), bv_cc -- TODO(jesse): 𝔹-valued eblast?
1766+
rw[pair_eq_pair_iff] at Hpr₁_right Hpr₂_right, auto_cases, -- , don't look at the tactic state
1767+
have := @H_ext i i' Γ_4 (by bv_cc), bv_cc -- TODO(): 𝔹-valued eblast?
17681768
end
17691769

17701770
lemma function.mk'_is_total {Γ} : Γ ≤ is_total x y (function.mk' F χ H_ext H_mem) :=
@@ -2009,12 +2009,12 @@ end
20092009
-- bv_split_at a_right_left_1, bv_split_at a_right_right_1,
20102010
-- simp only with cleanup at a_right_left_1_1_1 a_right_right_1_1_1,
20112011
-- bv_mp a_right_right_1_1_1 (eq_of_eq_pair_left),
2012-
-- bv_mp a_right_right_1_1_1 (eq_of_eq_pair_right), -- TODO(jesse) generate sane variable names
2012+
-- bv_mp a_right_right_1_1_1 (eq_of_eq_pair_right), -- TODO() generate sane variable names
20132013
-- bv_mp a_right_left_1_1_1 (eq_of_eq_pair_left),
20142014
-- bv_mp a_right_left_1_1_1 (eq_of_eq_pair_right),
20152015
-- have : Γ_2 ≤ func u i =ᴮ func u j, apply bv_trans, rw[bv_eq_symm],
20162016
-- assumption, rw[bv_eq_symm], apply bv_trans, rw[bv_eq_symm],
2017-
-- assumption, assumption, -- TODO(jesse) write a cc-like tactic to automate this
2017+
-- assumption, assumption, -- TODO() write a cc-like tactic to automate this
20182018
-- suffices : Γ_2 ≤ F i =ᴮ F j,
20192019
-- by {apply bv_trans, assumption, rw[bv_eq_symm], apply bv_trans,
20202020
-- assumption, from this},
@@ -2690,7 +2690,7 @@ begin
26902690
bv_cases_at H_mem k, cases k with k, simp at H_mem_1, refine bv_use _,
26912691
exact (ulift.up $ k + 1), simp, apply bv_rw' H_mem_1,
26922692
{ exact @B_ext_term 𝔹 _ (λ z, z =ᴮ ((k+1)̃ ̌)) succ (by simp) (by simp) },
2693-
-- TODO(jesse): automate calculation of the motive
2693+
-- TODO(): automate calculation of the motive
26942694
{ simp[pSet.of_nat, succ] },
26952695
end
26962696

src/henkin.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -128,7 +128,7 @@ def diagram.mk.map {F : ℕ → Language} {h_succ : ∀{i : ℕ}, F i →ᴸ F (
128128
| x (y+1) h := by {by_cases x = y + 1, rw[h], exact ⟨λn, id, λn, id⟩, refine h_succ ∘ _,
129129
apply diagram.mk.map, apply nat.le_of_le_and_ne_succ, repeat{assumption}}
130130

131-
--TODO(jesse) finish converting this to language versions and refactor henkin_language_chain
131+
--TODO() finish converting this to language versions and refactor henkin_language_chain
132132
-- @[simp]lemma diagram.mk.map_self_id {F : ℕ → Type*} {h_succ : ∀(i : ℕ), F i → F (i+1)} (x : ℕ) :
133133
-- @diagram.mk.map F @h_succ x x (by constructor) = id :=
134134
-- by {induction x, tidy, simp[diagram.mk.map,*], refl}
@@ -504,7 +504,7 @@ end
504504
-- to complete the structural recursion
505505

506506
/- The universal map from colimit preterm L_n → preterm L_infty is a bijection -/
507-
-- TODO(jesse) refactor with new colimit lemmas
507+
-- TODO() refactor with new colimit lemmas
508508
lemma term_comparison_bijective {L : Language} (l) : function.bijective (@term_comparison L l) :=
509509
begin
510510
refine ⟨_,_⟩,
@@ -880,7 +880,7 @@ end
880880
-- have : ∃ k : ℕ, @ι L T k ⊢' bd_falsum,
881881
-- {sorry}, -- again, this depends on picking a representative of a germ-eq class
882882
-- -- on the induced colimit of formulas
883-
-- -- remark(Floris): we need a lemma that if a directed union of theories proves f, then an element of it proves f.
883+
-- -- remark(): we need a lemma that if a directed union of theories proves f, then an element of it proves f.
884884
-- cases this with k P', unfold ι at P',
885885
-- apply is_consistent_henkin_theory_chain hT k,
886886
-- apply nonempty.map (Lhom.reflect_prf (henkin_language_canonical_map_inj k)),

src/pSet_ordinal.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1049,7 +1049,7 @@ lemma powerset_sound {x : pSet.{u}} : ⟦pSet.powerset x⟧ = Set.powerset ⟦x
10491049
def set_of_indicator {x : pSet.{u}} (χ : x.type → Prop) : pSet.{u} :=
10501050
⟨{i // χ i}, λ p, x.func (p.1)⟩
10511051

1052-
def functions (x y : pSet.{u}) : pSet.{u} := -- TODO(jesse): show this satisfies specification
1052+
def functions (x y : pSet.{u}) : pSet.{u} := -- TODO(): show this satisfies specification
10531053
@set_of_indicator (powerset $ prod x y)
10541054
(λ i_S, is_func x y ((powerset $ prod x y).func i_S))
10551055

src/parse_formula.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1,7 +1,7 @@
11
/-
22
Copyright (c) 2019 The Flypitch Project. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
4-
Author(s): Jesse Michael Han, Floris van Doorn
4+
Author(s):
55
66
Parsing formulas from Lean expressions.
77
-/
@@ -71,7 +71,7 @@ meta def to_term_empty : Π {n : ℕ}, expr → option (preterm L_empty n)
7171
| 0 (expr.var k) := some (var k)
7272
| _ _ := none
7373

74-
-- TODO(jesse) insert a case analysis on whether e' : Prop to determine whether or not to use imp
74+
-- TODO() insert a case analysis on whether e' : Prop to determine whether or not to use imp
7575
meta def to_formula_empty : Π {n : ℕ}, expr → option (preformula L_empty n)
7676
| 0 (expr.pi _ _ e' e) := ((to_formula_empty e) >>= (λ f, return (all f)))
7777
| 0 `(%%a = %%b) := do e₁ <- to_term_empty a, e₂ <- to_term_empty b,

src/print_formula.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -53,7 +53,7 @@ meta def print_formula : ∀ {n : ℕ}, bounded_formula L_ZFC n → string := λ
5353

5454
meta def print_formula_list {n} (axms : list (bounded_formula L_ZFC n)) : tactic unit :=
5555
do tactic.trace (to_string axms)
56-
-- TODO(jesse) format this so that newlines are inserted after commas
56+
-- TODO() format this so that newlines are inserted after commas
5757

5858
section test
5959

src/to_mathlib.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -1313,7 +1313,7 @@ do v_a <- target >>= lhs_of_le,
13131313
Γ_name <- get_unused_name "Γ",
13141314
v <- mk_mvar, v' <- mk_mvar,
13151315
Γ_new <- pose Γ_name none v,
1316-
-- TODO(jesse) try replacing to_expr with an expression via mk_app instead
1316+
-- TODO() try replacing to_expr with an expression via mk_app instead
13171317
new_goal <- to_expr ``((%%Γ_new : %%tp) ≤ %%v'),
13181318
tactic.change new_goal,
13191319
ctx <- local_context,
@@ -1334,7 +1334,7 @@ do v_a <- target >>= lhs_of_le,
13341334
Γ_name <- get_unused_name "Γ",
13351335
v <- mk_mvar, v' <- mk_mvar,
13361336
Γ_new <- pose Γ_name none v,
1337-
-- TODO(jesse) try replacing to_expr with an expression via mk_app instead
1337+
-- TODO() try replacing to_expr with an expression via mk_app instead
13381338
new_goal <- to_expr ``((%%Γ_new : %%tp) ≤ %%v'),
13391339
tactic.change new_goal,
13401340
ctx <- local_context,
@@ -1355,7 +1355,7 @@ do v_a <- target >>= lhs_of_le,
13551355
Γ_name <- get_unused_name "Γ",
13561356
v <- mk_mvar, v' <- mk_mvar,
13571357
Γ_new <- pose Γ_name none v,
1358-
-- TODO(jesse) try replacing to_expr with an expression via mk_app instead
1358+
-- TODO() try replacing to_expr with an expression via mk_app instead
13591359
new_goal <- to_expr ``((%%Γ_new : %%tp) ≤ %%v'),
13601360
tactic.change new_goal,
13611361
ctx <- local_context,
@@ -1477,7 +1477,7 @@ begin
14771477
{ by simp* }
14781478
end
14791479

1480-
-- TODO(jesse) debug these
1480+
-- TODO() debug these
14811481
-- meta def auto_or_elim_step : tactic unit :=
14821482
-- do ctx <- local_context >>= (λ l, l.mfilter hyp_is_ineq_sup),
14831483
-- if ctx.length > 0 then

0 commit comments

Comments
 (0)