url
stringclasses
147 values
commit
stringclasses
147 values
file_path
stringlengths
7
101
full_name
stringlengths
1
94
start
stringlengths
6
10
end
stringlengths
6
11
tactic
stringlengths
1
11.2k
state_before
stringlengths
3
2.09M
state_after
stringlengths
6
2.09M
https://github.com/MichaelStollBayreuth/EulerProducts.git
21e07835d1a467b99b5c3c9390d61ae69404445d
EulerProducts/PNT.lean
PNT_vonMangoldt
[438, 1]
[451, 10]
refine continuousOn_neg_logDeriv_ζ₁.mono fun s _ ↦ ?_
case refine_2 WIT : WienerIkeharaTheorem hnv : ∀ ⦃z : ℂ⦄, z ≠ 1 → 1 ≤ z.re → ζ z ≠ 0 ⊢ ContinuousOn (fun z => -deriv ζ₁ z / ζ₁ z) {s | 1 ≤ s.re}
case refine_2 WIT : WienerIkeharaTheorem hnv : ∀ ⦃z : ℂ⦄, z ≠ 1 → 1 ≤ z.re → ζ z ≠ 0 s : ℂ x✝ : s ∈ {s | 1 ≤ s.re} ⊢ s ∈ {z | z = 1 ∨ ζ z ≠ 0}
https://github.com/MichaelStollBayreuth/EulerProducts.git
21e07835d1a467b99b5c3c9390d61ae69404445d
EulerProducts/PNT.lean
PNT_vonMangoldt
[438, 1]
[451, 10]
specialize @hnv s
case refine_2 WIT : WienerIkeharaTheorem hnv : ∀ ⦃z : ℂ⦄, z ≠ 1 → 1 ≤ z.re → ζ z ≠ 0 s : ℂ x✝ : s ∈ {s | 1 ≤ s.re} ⊢ s ∈ {z | z = 1 ∨ ζ z ≠ 0}
case refine_2 WIT : WienerIkeharaTheorem s : ℂ x✝ : s ∈ {s | 1 ≤ s.re} hnv : s ≠ 1 → 1 ≤ s.re → ζ s ≠ 0 ⊢ s ∈ {z | z = 1 ∨ ζ z ≠ 0}
https://github.com/MichaelStollBayreuth/EulerProducts.git
21e07835d1a467b99b5c3c9390d61ae69404445d
EulerProducts/PNT.lean
PNT_vonMangoldt
[438, 1]
[451, 10]
simp at *
case refine_2 WIT : WienerIkeharaTheorem s : ℂ x✝ : s ∈ {s | 1 ≤ s.re} hnv : s ≠ 1 → 1 ≤ s.re → ζ s ≠ 0 ⊢ s ∈ {z | z = 1 ∨ ζ z ≠ 0}
case refine_2 WIT : WienerIkeharaTheorem s : ℂ x✝ : 1 ≤ s.re hnv : ¬s = 1 → 1 ≤ s.re → ¬ζ s = 0 ⊢ s = 1 ∨ ¬ζ s = 0
https://github.com/MichaelStollBayreuth/EulerProducts.git
21e07835d1a467b99b5c3c9390d61ae69404445d
EulerProducts/PNT.lean
PNT_vonMangoldt
[438, 1]
[451, 10]
tauto
case refine_2 WIT : WienerIkeharaTheorem s : ℂ x✝ : 1 ≤ s.re hnv : ¬s = 1 → 1 ≤ s.re → ¬ζ s = 0 ⊢ s = 1 ∨ ¬ζ s = 0
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.prop_left
[26, 9]
[31, 12]
intro h
P✝ : Sort u_1 A : Typ P✝ B : Bunch P✝ ⊢ ¬PreEquiv (prop A) B
P✝ : Sort u_1 A : Typ P✝ B : Bunch P✝ h : PreEquiv (prop A) B ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.prop_left
[26, 9]
[31, 12]
generalize hA' : prop A = A' at h
P✝ : Sort u_1 A : Typ P✝ B : Bunch P✝ h : PreEquiv (prop A) B ⊢ False
P✝ : Sort u_1 A : Typ P✝ B A' : Bunch P✝ hA' : prop A = A' h : PreEquiv A' B ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.prop_left
[26, 9]
[31, 12]
induction h <;> simp at hA'
P✝ : Sort u_1 A : Typ P✝ B A' : Bunch P✝ hA' : prop A = A' h : PreEquiv A' B ⊢ False
case subbunch P✝ : Sort u_1 A : Typ P✝ B A' : Bunch P✝ h✝ : BunchWithHole P✝ b1✝ b2✝ : Bunch P✝ a✝ : PreEquiv b1✝ b2✝ a_ih✝ : prop A = b1✝ → False hA' : h✝ = BunchWithHole.hole ∧ b1✝ = prop A ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.prop_left
[26, 9]
[31, 12]
rcases hA' with ⟨rfl,rfl⟩
case subbunch P✝ : Sort u_1 A : Typ P✝ B A' : Bunch P✝ h✝ : BunchWithHole P✝ b1✝ b2✝ : Bunch P✝ a✝ : PreEquiv b1✝ b2✝ a_ih✝ : prop A = b1✝ → False hA' : h✝ = BunchWithHole.hole ∧ b1✝ = prop A ⊢ False
case subbunch.intro P✝ : Sort u_1 A : Typ P✝ B A' b2✝ : Bunch P✝ a✝ : PreEquiv (prop A) b2✝ a_ih✝ : prop A = prop A → False ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.prop_left
[26, 9]
[31, 12]
simp at *
case subbunch.intro P✝ : Sort u_1 A : Typ P✝ B A' b2✝ : Bunch P✝ a✝ : PreEquiv (prop A) b2✝ a_ih✝ : prop A = prop A → False ⊢ False
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.sunit_left
[33, 9]
[38, 12]
intro h
P✝ : Sort u_1 B : Bunch P✝ ⊢ ¬PreEquiv sunit B
P✝ : Sort u_1 B : Bunch P✝ h : PreEquiv sunit B ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.sunit_left
[33, 9]
[38, 12]
generalize hA' : sunit = A' at h
P✝ : Sort u_1 B : Bunch P✝ h : PreEquiv sunit B ⊢ False
P✝ : Sort u_1 B A' : Bunch P✝ hA' : sunit = A' h : PreEquiv A' B ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.sunit_left
[33, 9]
[38, 12]
induction h <;> simp at hA'
P✝ : Sort u_1 B A' : Bunch P✝ hA' : sunit = A' h : PreEquiv A' B ⊢ False
case subbunch P✝ : Sort u_1 B A' : Bunch P✝ h✝ : BunchWithHole P✝ b1✝ b2✝ : Bunch P✝ a✝ : PreEquiv b1✝ b2✝ a_ih✝ : sunit = b1✝ → False hA' : h✝ = BunchWithHole.hole ∧ b1✝ = sunit ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.sunit_left
[33, 9]
[38, 12]
rcases hA' with ⟨rfl,rfl⟩
case subbunch P✝ : Sort u_1 B A' : Bunch P✝ h✝ : BunchWithHole P✝ b1✝ b2✝ : Bunch P✝ a✝ : PreEquiv b1✝ b2✝ a_ih✝ : sunit = b1✝ → False hA' : h✝ = BunchWithHole.hole ∧ b1✝ = sunit ⊢ False
case subbunch.intro P✝ : Sort u_1 B A' b2✝ : Bunch P✝ a✝ : PreEquiv sunit b2✝ a_ih✝ : sunit = sunit → False ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.sunit_left
[33, 9]
[38, 12]
simp at *
case subbunch.intro P✝ : Sort u_1 B A' b2✝ : Bunch P✝ a✝ : PreEquiv sunit b2✝ a_ih✝ : sunit = sunit → False ⊢ False
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.cunit_left
[40, 9]
[45, 12]
intro h
P✝ : Sort u_1 B : Bunch P✝ ⊢ ¬PreEquiv cunit B
P✝ : Sort u_1 B : Bunch P✝ h : PreEquiv cunit B ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.cunit_left
[40, 9]
[45, 12]
generalize hA' : cunit = A' at h
P✝ : Sort u_1 B : Bunch P✝ h : PreEquiv cunit B ⊢ False
P✝ : Sort u_1 B A' : Bunch P✝ hA' : cunit = A' h : PreEquiv A' B ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.cunit_left
[40, 9]
[45, 12]
induction h <;> simp at hA'
P✝ : Sort u_1 B A' : Bunch P✝ hA' : cunit = A' h : PreEquiv A' B ⊢ False
case subbunch P✝ : Sort u_1 B A' : Bunch P✝ h✝ : BunchWithHole P✝ b1✝ b2✝ : Bunch P✝ a✝ : PreEquiv b1✝ b2✝ a_ih✝ : cunit = b1✝ → False hA' : h✝ = BunchWithHole.hole ∧ b1✝ = cunit ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.cunit_left
[40, 9]
[45, 12]
rcases hA' with ⟨rfl,rfl⟩
case subbunch P✝ : Sort u_1 B A' : Bunch P✝ h✝ : BunchWithHole P✝ b1✝ b2✝ : Bunch P✝ a✝ : PreEquiv b1✝ b2✝ a_ih✝ : cunit = b1✝ → False hA' : h✝ = BunchWithHole.hole ∧ b1✝ = cunit ⊢ False
case subbunch.intro P✝ : Sort u_1 B A' b2✝ : Bunch P✝ a✝ : PreEquiv cunit b2✝ a_ih✝ : cunit = cunit → False ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.cunit_left
[40, 9]
[45, 12]
simp at *
case subbunch.intro P✝ : Sort u_1 B A' b2✝ : Bunch P✝ a✝ : PreEquiv cunit b2✝ a_ih✝ : cunit = cunit → False ⊢ False
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.prop_right
[47, 9]
[61, 19]
constructor
P✝ : Sort u_1 B : Bunch P✝ A : Typ P✝ ⊢ PreEquiv B (prop A) ↔ B = (cunit ,ᵇ prop A) ∨ B = (prop A ,ᵇ cunit) ∨ B = (sunit ;ᵇ prop A) ∨ B = (prop A ;ᵇ sunit)
case mp P✝ : Sort u_1 B : Bunch P✝ A : Typ P✝ ⊢ PreEquiv B (prop A) → B = (cunit ,ᵇ prop A) ∨ B = (prop A ,ᵇ cunit) ∨ B = (sunit ;ᵇ prop A) ∨ B = (prop A ;ᵇ sunit) case mpr P✝ : Sort u_1 B : Bunch P✝ A : Typ P✝ ⊢ B = (cunit ,ᵇ prop A) ∨ B = (prop A ,ᵇ cunit) ∨ B = (sunit ;ᵇ prop A) ∨ B = (prop A ;ᵇ sunit) → PreEquiv B (prop A)
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.prop_right
[47, 9]
[61, 19]
intro h
case mp P✝ : Sort u_1 B : Bunch P✝ A : Typ P✝ ⊢ PreEquiv B (prop A) → B = (cunit ,ᵇ prop A) ∨ B = (prop A ,ᵇ cunit) ∨ B = (sunit ;ᵇ prop A) ∨ B = (prop A ;ᵇ sunit)
case mp P✝ : Sort u_1 B : Bunch P✝ A : Typ P✝ h : PreEquiv B (prop A) ⊢ B = (cunit ,ᵇ prop A) ∨ B = (prop A ,ᵇ cunit) ∨ B = (sunit ;ᵇ prop A) ∨ B = (prop A ;ᵇ sunit)
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.prop_right
[47, 9]
[61, 19]
generalize hA' : prop A = A' at h
case mp P✝ : Sort u_1 B : Bunch P✝ A : Typ P✝ h : PreEquiv B (prop A) ⊢ B = (cunit ,ᵇ prop A) ∨ B = (prop A ,ᵇ cunit) ∨ B = (sunit ;ᵇ prop A) ∨ B = (prop A ;ᵇ sunit)
case mp P✝ : Sort u_1 B : Bunch P✝ A : Typ P✝ A' : Bunch P✝ hA' : prop A = A' h : PreEquiv B A' ⊢ B = (cunit ,ᵇ A') ∨ B = (A' ,ᵇ cunit) ∨ B = (sunit ;ᵇ A') ∨ B = (A' ;ᵇ sunit)
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.prop_right
[47, 9]
[61, 19]
induction h <;> simp_all
case mp P✝ : Sort u_1 B : Bunch P✝ A : Typ P✝ A' : Bunch P✝ hA' : prop A = A' h : PreEquiv B A' ⊢ B = (cunit ,ᵇ A') ∨ B = (A' ,ᵇ cunit) ∨ B = (sunit ;ᵇ A') ∨ B = (A' ;ᵇ sunit)
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.prop_right
[47, 9]
[61, 19]
rintro (rfl|rfl|rfl|rfl)
case mpr P✝ : Sort u_1 B : Bunch P✝ A : Typ P✝ ⊢ B = (cunit ,ᵇ prop A) ∨ B = (prop A ,ᵇ cunit) ∨ B = (sunit ;ᵇ prop A) ∨ B = (prop A ;ᵇ sunit) → PreEquiv B (prop A)
case mpr.inl P✝ : Sort u_1 A : Typ P✝ ⊢ PreEquiv (cunit ,ᵇ prop A) (prop A) case mpr.inr.inl P✝ : Sort u_1 A : Typ P✝ ⊢ PreEquiv (prop A ,ᵇ cunit) (prop A) case mpr.inr.inr.inl P✝ : Sort u_1 A : Typ P✝ ⊢ PreEquiv (sunit ;ᵇ prop A) (prop A) case mpr.inr.inr.inr P✝ : Sort u_1 A : Typ P✝ ⊢ PreEquiv (prop A ;ᵇ sunit) (prop A)
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.prop_right
[47, 9]
[61, 19]
exact cunitL
case mpr.inl P✝ : Sort u_1 A : Typ P✝ ⊢ PreEquiv (cunit ,ᵇ prop A) (prop A)
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.prop_right
[47, 9]
[61, 19]
exact cunitR
case mpr.inr.inl P✝ : Sort u_1 A : Typ P✝ ⊢ PreEquiv (prop A ,ᵇ cunit) (prop A)
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.prop_right
[47, 9]
[61, 19]
exact sunitL
case mpr.inr.inr.inl P✝ : Sort u_1 A : Typ P✝ ⊢ PreEquiv (sunit ;ᵇ prop A) (prop A)
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.prop_right
[47, 9]
[61, 19]
exact sunitR
case mpr.inr.inr.inr P✝ : Sort u_1 A : Typ P✝ ⊢ PreEquiv (prop A ;ᵇ sunit) (prop A)
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.sunit_right
[63, 9]
[77, 19]
constructor
P✝ : Sort u_1 B : Bunch P✝ ⊢ PreEquiv B sunit ↔ B = (cunit ,ᵇ sunit) ∨ B = (sunit ,ᵇ cunit) ∨ B = (sunit ;ᵇ sunit) ∨ B = (sunit ;ᵇ sunit)
case mp P✝ : Sort u_1 B : Bunch P✝ ⊢ PreEquiv B sunit → B = (cunit ,ᵇ sunit) ∨ B = (sunit ,ᵇ cunit) ∨ B = (sunit ;ᵇ sunit) ∨ B = (sunit ;ᵇ sunit) case mpr P✝ : Sort u_1 B : Bunch P✝ ⊢ B = (cunit ,ᵇ sunit) ∨ B = (sunit ,ᵇ cunit) ∨ B = (sunit ;ᵇ sunit) ∨ B = (sunit ;ᵇ sunit) → PreEquiv B sunit
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.sunit_right
[63, 9]
[77, 19]
intro h
case mp P✝ : Sort u_1 B : Bunch P✝ ⊢ PreEquiv B sunit → B = (cunit ,ᵇ sunit) ∨ B = (sunit ,ᵇ cunit) ∨ B = (sunit ;ᵇ sunit) ∨ B = (sunit ;ᵇ sunit)
case mp P✝ : Sort u_1 B : Bunch P✝ h : PreEquiv B sunit ⊢ B = (cunit ,ᵇ sunit) ∨ B = (sunit ,ᵇ cunit) ∨ B = (sunit ;ᵇ sunit) ∨ B = (sunit ;ᵇ sunit)
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.sunit_right
[63, 9]
[77, 19]
generalize hA' : sunit = A' at h
case mp P✝ : Sort u_1 B : Bunch P✝ h : PreEquiv B sunit ⊢ B = (cunit ,ᵇ sunit) ∨ B = (sunit ,ᵇ cunit) ∨ B = (sunit ;ᵇ sunit) ∨ B = (sunit ;ᵇ sunit)
case mp P✝ : Sort u_1 B A' : Bunch P✝ hA' : sunit = A' h : PreEquiv B A' ⊢ B = (cunit ,ᵇ A') ∨ B = (A' ,ᵇ cunit) ∨ B = (A' ;ᵇ A') ∨ B = (A' ;ᵇ A')
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.sunit_right
[63, 9]
[77, 19]
induction h <;> simp_all
case mp P✝ : Sort u_1 B A' : Bunch P✝ hA' : sunit = A' h : PreEquiv B A' ⊢ B = (cunit ,ᵇ A') ∨ B = (A' ,ᵇ cunit) ∨ B = (A' ;ᵇ A') ∨ B = (A' ;ᵇ A')
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.sunit_right
[63, 9]
[77, 19]
rintro (rfl|rfl|rfl|rfl)
case mpr P✝ : Sort u_1 B : Bunch P✝ ⊢ B = (cunit ,ᵇ sunit) ∨ B = (sunit ,ᵇ cunit) ∨ B = (sunit ;ᵇ sunit) ∨ B = (sunit ;ᵇ sunit) → PreEquiv B sunit
case mpr.inl P✝ : Sort u_1 ⊢ PreEquiv (cunit ,ᵇ sunit) sunit case mpr.inr.inl P✝ : Sort u_1 ⊢ PreEquiv (sunit ,ᵇ cunit) sunit case mpr.inr.inr.inl P✝ : Sort u_1 ⊢ PreEquiv (sunit ;ᵇ sunit) sunit case mpr.inr.inr.inr P✝ : Sort u_1 ⊢ PreEquiv (sunit ;ᵇ sunit) sunit
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.sunit_right
[63, 9]
[77, 19]
exact cunitL
case mpr.inl P✝ : Sort u_1 ⊢ PreEquiv (cunit ,ᵇ sunit) sunit
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.sunit_right
[63, 9]
[77, 19]
exact cunitR
case mpr.inr.inl P✝ : Sort u_1 ⊢ PreEquiv (sunit ,ᵇ cunit) sunit
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.sunit_right
[63, 9]
[77, 19]
exact sunitL
case mpr.inr.inr.inl P✝ : Sort u_1 ⊢ PreEquiv (sunit ;ᵇ sunit) sunit
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.sunit_right
[63, 9]
[77, 19]
exact sunitR
case mpr.inr.inr.inr P✝ : Sort u_1 ⊢ PreEquiv (sunit ;ᵇ sunit) sunit
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.cunit_right
[79, 9]
[93, 19]
constructor
P✝ : Sort u_1 B : Bunch P✝ ⊢ PreEquiv B cunit ↔ B = (cunit ,ᵇ cunit) ∨ B = (cunit ,ᵇ cunit) ∨ B = (sunit ;ᵇ cunit) ∨ B = (cunit ;ᵇ sunit)
case mp P✝ : Sort u_1 B : Bunch P✝ ⊢ PreEquiv B cunit → B = (cunit ,ᵇ cunit) ∨ B = (cunit ,ᵇ cunit) ∨ B = (sunit ;ᵇ cunit) ∨ B = (cunit ;ᵇ sunit) case mpr P✝ : Sort u_1 B : Bunch P✝ ⊢ B = (cunit ,ᵇ cunit) ∨ B = (cunit ,ᵇ cunit) ∨ B = (sunit ;ᵇ cunit) ∨ B = (cunit ;ᵇ sunit) → PreEquiv B cunit
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.cunit_right
[79, 9]
[93, 19]
intro h
case mp P✝ : Sort u_1 B : Bunch P✝ ⊢ PreEquiv B cunit → B = (cunit ,ᵇ cunit) ∨ B = (cunit ,ᵇ cunit) ∨ B = (sunit ;ᵇ cunit) ∨ B = (cunit ;ᵇ sunit)
case mp P✝ : Sort u_1 B : Bunch P✝ h : PreEquiv B cunit ⊢ B = (cunit ,ᵇ cunit) ∨ B = (cunit ,ᵇ cunit) ∨ B = (sunit ;ᵇ cunit) ∨ B = (cunit ;ᵇ sunit)
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.cunit_right
[79, 9]
[93, 19]
generalize hA' : cunit = A' at h
case mp P✝ : Sort u_1 B : Bunch P✝ h : PreEquiv B cunit ⊢ B = (cunit ,ᵇ cunit) ∨ B = (cunit ,ᵇ cunit) ∨ B = (sunit ;ᵇ cunit) ∨ B = (cunit ;ᵇ sunit)
case mp P✝ : Sort u_1 B A' : Bunch P✝ hA' : cunit = A' h : PreEquiv B A' ⊢ B = (A' ,ᵇ A') ∨ B = (A' ,ᵇ A') ∨ B = (sunit ;ᵇ A') ∨ B = (A' ;ᵇ sunit)
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.cunit_right
[79, 9]
[93, 19]
induction h <;> simp_all
case mp P✝ : Sort u_1 B A' : Bunch P✝ hA' : cunit = A' h : PreEquiv B A' ⊢ B = (A' ,ᵇ A') ∨ B = (A' ,ᵇ A') ∨ B = (sunit ;ᵇ A') ∨ B = (A' ;ᵇ sunit)
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.cunit_right
[79, 9]
[93, 19]
rintro (rfl|rfl|rfl|rfl)
case mpr P✝ : Sort u_1 B : Bunch P✝ ⊢ B = (cunit ,ᵇ cunit) ∨ B = (cunit ,ᵇ cunit) ∨ B = (sunit ;ᵇ cunit) ∨ B = (cunit ;ᵇ sunit) → PreEquiv B cunit
case mpr.inl P✝ : Sort u_1 ⊢ PreEquiv (cunit ,ᵇ cunit) cunit case mpr.inr.inl P✝ : Sort u_1 ⊢ PreEquiv (cunit ,ᵇ cunit) cunit case mpr.inr.inr.inl P✝ : Sort u_1 ⊢ PreEquiv (sunit ;ᵇ cunit) cunit case mpr.inr.inr.inr P✝ : Sort u_1 ⊢ PreEquiv (cunit ;ᵇ sunit) cunit
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.cunit_right
[79, 9]
[93, 19]
exact cunitL
case mpr.inl P✝ : Sort u_1 ⊢ PreEquiv (cunit ,ᵇ cunit) cunit
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.cunit_right
[79, 9]
[93, 19]
exact cunitR
case mpr.inr.inl P✝ : Sort u_1 ⊢ PreEquiv (cunit ,ᵇ cunit) cunit
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.cunit_right
[79, 9]
[93, 19]
exact sunitL
case mpr.inr.inr.inl P✝ : Sort u_1 ⊢ PreEquiv (sunit ;ᵇ cunit) cunit
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.PreEquiv.cunit_right
[79, 9]
[93, 19]
exact sunitR
case mpr.inr.inr.inr P✝ : Sort u_1 ⊢ PreEquiv (cunit ;ᵇ sunit) cunit
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.Equiv.subbunch
[127, 1]
[141, 24]
intro e
P : Type u_1 b1 b2 : Bunch P h : BunchWithHole P ⊢ b1 ≈ b2 → ↑h b1 ≈ ↑h b2
P : Type u_1 b1 b2 : Bunch P h : BunchWithHole P e : b1 ≈ b2 ⊢ ↑h b1 ≈ ↑h b2
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.Equiv.subbunch
[127, 1]
[141, 24]
induction e with | rel _ _ h => apply EqvGen.rel apply PreEquiv.subbunch exact h | refl => exact refl | symm _ _ _ ih => exact symm ih | trans _ _ _ _ _ ih1 ih2 => exact trans ih1 ih2
P : Type u_1 b1 b2 : Bunch P h : BunchWithHole P e : b1 ≈ b2 ⊢ ↑h b1 ≈ ↑h b2
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.Equiv.subbunch
[127, 1]
[141, 24]
apply EqvGen.rel
case rel P : Type u_1 b1 b2 : Bunch P h✝ : BunchWithHole P x✝ y✝ : Bunch P h : PreEquiv x✝ y✝ ⊢ ↑h✝ x✝ ≈ ↑h✝ y✝
case rel.a P : Type u_1 b1 b2 : Bunch P h✝ : BunchWithHole P x✝ y✝ : Bunch P h : PreEquiv x✝ y✝ ⊢ PreEquiv (↑h✝ x✝) (↑h✝ y✝)
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.Equiv.subbunch
[127, 1]
[141, 24]
apply PreEquiv.subbunch
case rel.a P : Type u_1 b1 b2 : Bunch P h✝ : BunchWithHole P x✝ y✝ : Bunch P h : PreEquiv x✝ y✝ ⊢ PreEquiv (↑h✝ x✝) (↑h✝ y✝)
case rel.a.a P : Type u_1 b1 b2 : Bunch P h✝ : BunchWithHole P x✝ y✝ : Bunch P h : PreEquiv x✝ y✝ ⊢ PreEquiv x✝ y✝
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.Equiv.subbunch
[127, 1]
[141, 24]
exact h
case rel.a.a P : Type u_1 b1 b2 : Bunch P h✝ : BunchWithHole P x✝ y✝ : Bunch P h : PreEquiv x✝ y✝ ⊢ PreEquiv x✝ y✝
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.Equiv.subbunch
[127, 1]
[141, 24]
exact refl
case refl P : Type u_1 b1 b2 : Bunch P h : BunchWithHole P x✝ : Bunch P ⊢ ↑h x✝ ≈ ↑h x✝
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.Equiv.subbunch
[127, 1]
[141, 24]
exact symm ih
case symm P : Type u_1 b1 b2 : Bunch P h : BunchWithHole P x✝ y✝ : Bunch P a✝ : EqvGen PreEquiv x✝ y✝ ih : ↑h x✝ ≈ ↑h y✝ ⊢ ↑h y✝ ≈ ↑h x✝
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.Equiv.subbunch
[127, 1]
[141, 24]
exact trans ih1 ih2
case trans P : Type u_1 b1 b2 : Bunch P h : BunchWithHole P x✝ y✝ z✝ : Bunch P a✝¹ : EqvGen PreEquiv x✝ y✝ a✝ : EqvGen PreEquiv y✝ z✝ ih1 : ↑h x✝ ≈ ↑h y✝ ih2 : ↑h y✝ ≈ ↑h z✝ ⊢ ↑h x✝ ≈ ↑h z✝
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.Equiv.hole_prop_inv
[157, 1]
[164, 8]
intro e
P : Type u_1 Γ : BunchWithHole P A : Typ P Δ : Bunch P ⊢ ↑Γ (prop A) ≈ Δ → ∃ Γ', Δ = ↑Γ' (prop A)
P : Type u_1 Γ : BunchWithHole P A : Typ P Δ : Bunch P e : ↑Γ (prop A) ≈ Δ ⊢ ∃ Γ', Δ = ↑Γ' (prop A)
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.Equiv.hole_prop_inv
[157, 1]
[164, 8]
induction Δ
P : Type u_1 Γ : BunchWithHole P A : Typ P Δ : Bunch P e : ↑Γ (prop A) ≈ Δ ⊢ ∃ Γ', Δ = ↑Γ' (prop A)
case prop P : Type u_1 Γ : BunchWithHole P A a✝ : Typ P e : ↑Γ (prop A) ≈ prop a✝ ⊢ ∃ Γ', prop a✝ = ↑Γ' (prop A) case cunit P : Type u_1 Γ : BunchWithHole P A : Typ P e : ↑Γ (prop A) ≈ cunit ⊢ ∃ Γ', cunit = ↑Γ' (prop A) case comma P : Type u_1 Γ : BunchWithHole P A : Typ P a✝¹ a✝ : Bunch P a_ih✝¹ : ↑Γ (prop A) ≈ a✝¹ → ∃ Γ', a✝¹ = ↑Γ' (prop A) a_ih✝ : ↑Γ (prop A) ≈ a✝ → ∃ Γ', a✝ = ↑Γ' (prop A) e : ↑Γ (prop A) ≈ (a✝¹ ,ᵇ a✝) ⊢ ∃ Γ', (a✝¹ ,ᵇ a✝) = ↑Γ' (prop A) case sunit P : Type u_1 Γ : BunchWithHole P A : Typ P e : ↑Γ (prop A) ≈ sunit ⊢ ∃ Γ', sunit = ↑Γ' (prop A) case semi P : Type u_1 Γ : BunchWithHole P A : Typ P a✝¹ a✝ : Bunch P a_ih✝¹ : ↑Γ (prop A) ≈ a✝¹ → ∃ Γ', a✝¹ = ↑Γ' (prop A) a_ih✝ : ↑Γ (prop A) ≈ a✝ → ∃ Γ', a✝ = ↑Γ' (prop A) e : ↑Γ (prop A) ≈ (a✝¹ ;ᵇ a✝) ⊢ ∃ Γ', (a✝¹ ;ᵇ a✝) = ↑Γ' (prop A)
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.Equiv.hole_prop_inv
[157, 1]
[164, 8]
case prop => simp at e refine ⟨.hole,?_⟩; simp
P : Type u_1 Γ : BunchWithHole P A a✝ : Typ P e : ↑Γ (prop A) ≈ prop a✝ ⊢ ∃ Γ', prop a✝ = ↑Γ' (prop A)
P : Type u_1 Γ : BunchWithHole P A a✝ : Typ P e : ↑Γ (prop A) ≈ prop a✝ ⊢ a✝ = A
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.Equiv.hole_prop_inv
[157, 1]
[164, 8]
sorry
case cunit P : Type u_1 Γ : BunchWithHole P A : Typ P e : ↑Γ (prop A) ≈ cunit ⊢ ∃ Γ', cunit = ↑Γ' (prop A) case comma P : Type u_1 Γ : BunchWithHole P A : Typ P a✝¹ a✝ : Bunch P a_ih✝¹ : ↑Γ (prop A) ≈ a✝¹ → ∃ Γ', a✝¹ = ↑Γ' (prop A) a_ih✝ : ↑Γ (prop A) ≈ a✝ → ∃ Γ', a✝ = ↑Γ' (prop A) e : ↑Γ (prop A) ≈ (a✝¹ ,ᵇ a✝) ⊢ ∃ Γ', (a✝¹ ,ᵇ a✝) = ↑Γ' (prop A) case sunit P : Type u_1 Γ : BunchWithHole P A : Typ P e : ↑Γ (prop A) ≈ sunit ⊢ ∃ Γ', sunit = ↑Γ' (prop A) case semi P : Type u_1 Γ : BunchWithHole P A : Typ P a✝¹ a✝ : Bunch P a_ih✝¹ : ↑Γ (prop A) ≈ a✝¹ → ∃ Γ', a✝¹ = ↑Γ' (prop A) a_ih✝ : ↑Γ (prop A) ≈ a✝ → ∃ Γ', a✝ = ↑Γ' (prop A) e : ↑Γ (prop A) ≈ (a✝¹ ;ᵇ a✝) ⊢ ∃ Γ', (a✝¹ ;ᵇ a✝) = ↑Γ' (prop A)
case comma P : Type u_1 Γ : BunchWithHole P A : Typ P a✝¹ a✝ : Bunch P a_ih✝¹ : ↑Γ (prop A) ≈ a✝¹ → ∃ Γ', a✝¹ = ↑Γ' (prop A) a_ih✝ : ↑Γ (prop A) ≈ a✝ → ∃ Γ', a✝ = ↑Γ' (prop A) e : ↑Γ (prop A) ≈ (a✝¹ ,ᵇ a✝) ⊢ ∃ Γ', (a✝¹ ,ᵇ a✝) = ↑Γ' (prop A) case sunit P : Type u_1 Γ : BunchWithHole P A : Typ P e : ↑Γ (prop A) ≈ sunit ⊢ ∃ Γ', sunit = ↑Γ' (prop A) case semi P : Type u_1 Γ : BunchWithHole P A : Typ P a✝¹ a✝ : Bunch P a_ih✝¹ : ↑Γ (prop A) ≈ a✝¹ → ∃ Γ', a✝¹ = ↑Γ' (prop A) a_ih✝ : ↑Γ (prop A) ≈ a✝ → ∃ Γ', a✝ = ↑Γ' (prop A) e : ↑Γ (prop A) ≈ (a✝¹ ;ᵇ a✝) ⊢ ∃ Γ', (a✝¹ ;ᵇ a✝) = ↑Γ' (prop A)
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.Equiv.hole_prop_inv
[157, 1]
[164, 8]
refine ⟨.hole,?_⟩
P : Type u_1 Γ : BunchWithHole P A a✝ : Typ P e : ↑Γ (prop A) ≈ prop a✝ ⊢ ∃ Γ', prop a✝ = ↑Γ' (prop A)
P : Type u_1 Γ : BunchWithHole P A a✝ : Typ P e : ↑Γ (prop A) ≈ prop a✝ ⊢ prop a✝ = ↑BunchWithHole.hole (prop A)
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Equiv.lean
BunchImpl.Equiv.hole_prop_inv
[157, 1]
[164, 8]
simp
P : Type u_1 Γ : BunchWithHole P A a✝ : Typ P e : ↑Γ (prop A) ≈ prop a✝ ⊢ prop a✝ = ↑BunchWithHole.hole (prop A)
P : Type u_1 Γ : BunchWithHole P A a✝ : Typ P e : ↑Γ (prop A) ≈ prop a✝ ⊢ a✝ = A
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.comma_eq_comma
[52, 9]
[56, 26]
constructor
P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ ⊢ (l1 ,ᵇ r1) = (l2 ,ᵇ r2) ↔ l1 = l2 ∧ r1 = r2
case mp P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ ⊢ (l1 ,ᵇ r1) = (l2 ,ᵇ r2) → l1 = l2 ∧ r1 = r2 case mpr P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ ⊢ l1 = l2 ∧ r1 = r2 → (l1 ,ᵇ r1) = (l2 ,ᵇ r2)
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.comma_eq_comma
[52, 9]
[56, 26]
intro h
case mp P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ ⊢ (l1 ,ᵇ r1) = (l2 ,ᵇ r2) → l1 = l2 ∧ r1 = r2
case mp P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ h : (l1 ,ᵇ r1) = (l2 ,ᵇ r2) ⊢ l1 = l2 ∧ r1 = r2
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.comma_eq_comma
[52, 9]
[56, 26]
constructor <;> (funext V; have := congrFun h V; simp at this; simp [*])
case mp P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ h : (l1 ,ᵇ r1) = (l2 ,ᵇ r2) ⊢ l1 = l2 ∧ r1 = r2
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.comma_eq_comma
[52, 9]
[56, 26]
funext V
case mp.right P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ h : (l1 ,ᵇ r1) = (l2 ,ᵇ r2) ⊢ r1 = r2
case mp.right.h P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ h : (l1 ,ᵇ r1) = (l2 ,ᵇ r2) V : Sort u_1 ⊢ r1 V = r2 V
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.comma_eq_comma
[52, 9]
[56, 26]
have := congrFun h V
case mp.right.h P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ h : (l1 ,ᵇ r1) = (l2 ,ᵇ r2) V : Sort u_1 ⊢ r1 V = r2 V
case mp.right.h P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ h : (l1 ,ᵇ r1) = (l2 ,ᵇ r2) V : Sort u_1 this : (l1 ,ᵇ r1) V = (l2 ,ᵇ r2) V ⊢ r1 V = r2 V
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.comma_eq_comma
[52, 9]
[56, 26]
simp at this
case mp.right.h P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ h : (l1 ,ᵇ r1) = (l2 ,ᵇ r2) V : Sort u_1 this : (l1 ,ᵇ r1) V = (l2 ,ᵇ r2) V ⊢ r1 V = r2 V
case mp.right.h P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ h : (l1 ,ᵇ r1) = (l2 ,ᵇ r2) V : Sort u_1 this : l1 V = l2 V ∧ r1 V = r2 V ⊢ r1 V = r2 V
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.comma_eq_comma
[52, 9]
[56, 26]
simp [*]
case mp.right.h P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ h : (l1 ,ᵇ r1) = (l2 ,ᵇ r2) V : Sort u_1 this : l1 V = l2 V ∧ r1 V = r2 V ⊢ r1 V = r2 V
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.comma_eq_comma
[52, 9]
[56, 26]
rintro ⟨rfl,rfl⟩
case mpr P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ ⊢ l1 = l2 ∧ r1 = r2 → (l1 ,ᵇ r1) = (l2 ,ᵇ r2)
case mpr.intro P✝ : Sort u_1 l1 r1 : Bunch P✝ ⊢ (l1 ,ᵇ r1) = (l1 ,ᵇ r1)
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.comma_eq_comma
[52, 9]
[56, 26]
rfl
case mpr.intro P✝ : Sort u_1 l1 r1 : Bunch P✝ ⊢ (l1 ,ᵇ r1) = (l1 ,ᵇ r1)
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.semi_eq_semi
[58, 9]
[62, 26]
constructor
P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ ⊢ (l1 ;ᵇ r1) = (l2 ;ᵇ r2) ↔ l1 = l2 ∧ r1 = r2
case mp P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ ⊢ (l1 ;ᵇ r1) = (l2 ;ᵇ r2) → l1 = l2 ∧ r1 = r2 case mpr P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ ⊢ l1 = l2 ∧ r1 = r2 → (l1 ;ᵇ r1) = (l2 ;ᵇ r2)
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.semi_eq_semi
[58, 9]
[62, 26]
intro h
case mp P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ ⊢ (l1 ;ᵇ r1) = (l2 ;ᵇ r2) → l1 = l2 ∧ r1 = r2
case mp P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ h : (l1 ;ᵇ r1) = (l2 ;ᵇ r2) ⊢ l1 = l2 ∧ r1 = r2
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.semi_eq_semi
[58, 9]
[62, 26]
constructor <;> (funext V; have := congrFun h V; simp at this; simp [*])
case mp P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ h : (l1 ;ᵇ r1) = (l2 ;ᵇ r2) ⊢ l1 = l2 ∧ r1 = r2
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.semi_eq_semi
[58, 9]
[62, 26]
funext V
case mp.right P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ h : (l1 ;ᵇ r1) = (l2 ;ᵇ r2) ⊢ r1 = r2
case mp.right.h P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ h : (l1 ;ᵇ r1) = (l2 ;ᵇ r2) V : Sort u_1 ⊢ r1 V = r2 V
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.semi_eq_semi
[58, 9]
[62, 26]
have := congrFun h V
case mp.right.h P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ h : (l1 ;ᵇ r1) = (l2 ;ᵇ r2) V : Sort u_1 ⊢ r1 V = r2 V
case mp.right.h P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ h : (l1 ;ᵇ r1) = (l2 ;ᵇ r2) V : Sort u_1 this : (l1 ;ᵇ r1) V = (l2 ;ᵇ r2) V ⊢ r1 V = r2 V
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.semi_eq_semi
[58, 9]
[62, 26]
simp at this
case mp.right.h P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ h : (l1 ;ᵇ r1) = (l2 ;ᵇ r2) V : Sort u_1 this : (l1 ;ᵇ r1) V = (l2 ;ᵇ r2) V ⊢ r1 V = r2 V
case mp.right.h P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ h : (l1 ;ᵇ r1) = (l2 ;ᵇ r2) V : Sort u_1 this : l1 V = l2 V ∧ r1 V = r2 V ⊢ r1 V = r2 V
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.semi_eq_semi
[58, 9]
[62, 26]
simp [*]
case mp.right.h P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ h : (l1 ;ᵇ r1) = (l2 ;ᵇ r2) V : Sort u_1 this : l1 V = l2 V ∧ r1 V = r2 V ⊢ r1 V = r2 V
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.semi_eq_semi
[58, 9]
[62, 26]
rintro ⟨rfl,rfl⟩
case mpr P✝ : Sort u_1 l1 r1 l2 r2 : Bunch P✝ ⊢ l1 = l2 ∧ r1 = r2 → (l1 ;ᵇ r1) = (l2 ;ᵇ r2)
case mpr.intro P✝ : Sort u_1 l1 r1 : Bunch P✝ ⊢ (l1 ;ᵇ r1) = (l1 ;ᵇ r1)
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.semi_eq_semi
[58, 9]
[62, 26]
rfl
case mpr.intro P✝ : Sort u_1 l1 r1 : Bunch P✝ ⊢ (l1 ;ᵇ r1) = (l1 ;ᵇ r1)
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_left_comma
[64, 9]
[70, 11]
intro h
P : Sort u b1 b2 : Bunch P ⊢ (b1 ,ᵇ b2) ≠ b1
P : Sort u b1 b2 : Bunch P h : (b1 ,ᵇ b2) = b1 ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_left_comma
[64, 9]
[70, 11]
have := congrArg sizeOf h
P : Sort u b1 b2 : Bunch P h : (b1 ,ᵇ b2) = b1 ⊢ False
P : Sort u b1 b2 : Bunch P h : (b1 ,ᵇ b2) = b1 this : sizeOf (b1 ,ᵇ b2) = sizeOf b1 ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_left_comma
[64, 9]
[70, 11]
clear h
P : Sort u b1 b2 : Bunch P h : (b1 ,ᵇ b2) = b1 this : sizeOf (b1 ,ᵇ b2) = sizeOf b1 ⊢ False
P : Sort u b1 b2 : Bunch P this : sizeOf (b1 ,ᵇ b2) = sizeOf b1 ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_left_comma
[64, 9]
[70, 11]
simp [instSizeOfBunch, comma] at this
P : Sort u b1 b2 : Bunch P this : sizeOf (b1 ,ᵇ b2) = sizeOf b1 ⊢ False
P : Sort u b1 b2 : Bunch P this : 1 + sizeOf (b1 PUnit.{u}) + sizeOf (b2 PUnit.{u}) = sizeOf (b1 PUnit.{u}) ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_left_comma
[64, 9]
[70, 11]
linarith
P : Sort u b1 b2 : Bunch P this : 1 + sizeOf (b1 PUnit.{u}) + sizeOf (b2 PUnit.{u}) = sizeOf (b1 PUnit.{u}) ⊢ False
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_right_comma
[72, 9]
[75, 40]
intro h
P✝ : Sort u_1 b1 b2 : Bunch P✝ ⊢ (b1 ,ᵇ b2) ≠ b2
P✝ : Sort u_1 b1 b2 : Bunch P✝ h : (b1 ,ᵇ b2) = b2 ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_right_comma
[72, 9]
[75, 40]
have := congrArg sizeOf h
P✝ : Sort u_1 b1 b2 : Bunch P✝ h : (b1 ,ᵇ b2) = b2 ⊢ False
P✝ : Sort u_1 b1 b2 : Bunch P✝ h : (b1 ,ᵇ b2) = b2 this : sizeOf (b1 ,ᵇ b2) = sizeOf b2 ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_right_comma
[72, 9]
[75, 40]
clear h
P✝ : Sort u_1 b1 b2 : Bunch P✝ h : (b1 ,ᵇ b2) = b2 this : sizeOf (b1 ,ᵇ b2) = sizeOf b2 ⊢ False
P✝ : Sort u_1 b1 b2 : Bunch P✝ this : sizeOf (b1 ,ᵇ b2) = sizeOf b2 ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_right_comma
[72, 9]
[75, 40]
simp [instSizeOfBunch, comma] at this
P✝ : Sort u_1 b1 b2 : Bunch P✝ this : sizeOf (b1 ,ᵇ b2) = sizeOf b2 ⊢ False
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_self_left_comma
[77, 9]
[81, 11]
intro h
P✝ : Sort u_1 b1 b2 : Bunch P✝ ⊢ b1 ≠ (b1 ,ᵇ b2)
P✝ : Sort u_1 b1 b2 : Bunch P✝ h : b1 = (b1 ,ᵇ b2) ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_self_left_comma
[77, 9]
[81, 11]
have := congrArg sizeOf h
P✝ : Sort u_1 b1 b2 : Bunch P✝ h : b1 = (b1 ,ᵇ b2) ⊢ False
P✝ : Sort u_1 b1 b2 : Bunch P✝ h : b1 = (b1 ,ᵇ b2) this : sizeOf b1 = sizeOf (b1 ,ᵇ b2) ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_self_left_comma
[77, 9]
[81, 11]
clear h
P✝ : Sort u_1 b1 b2 : Bunch P✝ h : b1 = (b1 ,ᵇ b2) this : sizeOf b1 = sizeOf (b1 ,ᵇ b2) ⊢ False
P✝ : Sort u_1 b1 b2 : Bunch P✝ this : sizeOf b1 = sizeOf (b1 ,ᵇ b2) ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_self_left_comma
[77, 9]
[81, 11]
simp [instSizeOfBunch, comma] at this
P✝ : Sort u_1 b1 b2 : Bunch P✝ this : sizeOf b1 = sizeOf (b1 ,ᵇ b2) ⊢ False
P✝ : Sort u_1 b1 b2 : Bunch P✝ this : sizeOf (b1 PUnit.{u_1}) = 1 + sizeOf (b1 PUnit.{u_1}) + sizeOf (b2 PUnit.{u_1}) ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_self_left_comma
[77, 9]
[81, 11]
linarith
P✝ : Sort u_1 b1 b2 : Bunch P✝ this : sizeOf (b1 PUnit.{u_1}) = 1 + sizeOf (b1 PUnit.{u_1}) + sizeOf (b2 PUnit.{u_1}) ⊢ False
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_self_right_comma
[83, 9]
[86, 40]
intro h
P✝ : Sort u_1 b2 b1 : Bunch P✝ ⊢ b2 ≠ (b1 ,ᵇ b2)
P✝ : Sort u_1 b2 b1 : Bunch P✝ h : b2 = (b1 ,ᵇ b2) ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_self_right_comma
[83, 9]
[86, 40]
have := congrArg sizeOf h
P✝ : Sort u_1 b2 b1 : Bunch P✝ h : b2 = (b1 ,ᵇ b2) ⊢ False
P✝ : Sort u_1 b2 b1 : Bunch P✝ h : b2 = (b1 ,ᵇ b2) this : sizeOf b2 = sizeOf (b1 ,ᵇ b2) ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_self_right_comma
[83, 9]
[86, 40]
clear h
P✝ : Sort u_1 b2 b1 : Bunch P✝ h : b2 = (b1 ,ᵇ b2) this : sizeOf b2 = sizeOf (b1 ,ᵇ b2) ⊢ False
P✝ : Sort u_1 b2 b1 : Bunch P✝ this : sizeOf b2 = sizeOf (b1 ,ᵇ b2) ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_self_right_comma
[83, 9]
[86, 40]
simp [instSizeOfBunch, comma] at this
P✝ : Sort u_1 b2 b1 : Bunch P✝ this : sizeOf b2 = sizeOf (b1 ,ᵇ b2) ⊢ False
no goals
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_left_semi
[88, 9]
[92, 11]
intro h
P✝ : Sort u_1 b1 b2 : Bunch P✝ ⊢ (b1 ;ᵇ b2) ≠ b1
P✝ : Sort u_1 b1 b2 : Bunch P✝ h : (b1 ;ᵇ b2) = b1 ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_left_semi
[88, 9]
[92, 11]
have := congrArg sizeOf h
P✝ : Sort u_1 b1 b2 : Bunch P✝ h : (b1 ;ᵇ b2) = b1 ⊢ False
P✝ : Sort u_1 b1 b2 : Bunch P✝ h : (b1 ;ᵇ b2) = b1 this : sizeOf (b1 ;ᵇ b2) = sizeOf b1 ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_left_semi
[88, 9]
[92, 11]
clear h
P✝ : Sort u_1 b1 b2 : Bunch P✝ h : (b1 ;ᵇ b2) = b1 this : sizeOf (b1 ;ᵇ b2) = sizeOf b1 ⊢ False
P✝ : Sort u_1 b1 b2 : Bunch P✝ this : sizeOf (b1 ;ᵇ b2) = sizeOf b1 ⊢ False
https://github.com/JamesGallicchio/brunched-invitations.git
3082c5ae68d2022b1439310f315a0038dae24e0c
BunchImpl/Term/Bunch.lean
BunchImpl.Bunch.neq_left_semi
[88, 9]
[92, 11]
simp [instSizeOfBunch, semi] at this
P✝ : Sort u_1 b1 b2 : Bunch P✝ this : sizeOf (b1 ;ᵇ b2) = sizeOf b1 ⊢ False
P✝ : Sort u_1 b1 b2 : Bunch P✝ this : 1 + sizeOf (b1 PUnit.{u_1}) + sizeOf (b2 PUnit.{u_1}) = sizeOf (b1 PUnit.{u_1}) ⊢ False