Skip to content

Commit

Permalink
Delete ToMathlib/Logic/Basic
Browse files Browse the repository at this point in the history
We no longer need `forall₂_and_distrib`, `forall_and` works.
  • Loading branch information
urkud committed Aug 1, 2024
1 parent a344c1b commit 62ac547
Show file tree
Hide file tree
Showing 3 changed files with 2 additions and 10 deletions.
1 change: 0 additions & 1 deletion SphereEversion.lean
Original file line number Diff line number Diff line change
Expand Up @@ -53,7 +53,6 @@ import SphereEversion.ToMathlib.Geometry.Manifold.VectorBundle.Misc
import SphereEversion.ToMathlib.LinearAlgebra.Basic
import SphereEversion.ToMathlib.LinearAlgebra.Basis
import SphereEversion.ToMathlib.LinearAlgebra.FiniteDimensional
import SphereEversion.ToMathlib.Logic.Basic
import SphereEversion.ToMathlib.MeasureTheory.BorelSpace
import SphereEversion.ToMathlib.MeasureTheory.ParametricIntervalIntegral
import SphereEversion.ToMathlib.Order.Filter.Basic
Expand Down
5 changes: 2 additions & 3 deletions SphereEversion/Global/Gromov.lean
Original file line number Diff line number Diff line change
@@ -1,7 +1,6 @@
import SphereEversion.Global.LocalisationData
import SphereEversion.Global.LocalizedConstruction
import SphereEversion.Global.ParametricityForFree
import SphereEversion.ToMathlib.Logic.Basic
import SphereEversion.ToMathlib.Geometry.Manifold.Metrizable

/-!
Expand Down Expand Up @@ -170,7 +169,7 @@ theorem RelMfld.Ample.satisfiesHPrinciple' (hRample : R.Ample) (hRopen : IsOpen
· apply hF'₁.mono fun x hx ↦ ?_
rw [hx]
rcases inductive_htpy_construction' P₀ P₁ P₂ hP₂ hP₂' init ind with ⟨F, hF₀, hFP₀, hFP₁, hFP₂⟩
simp only [P₀, forall₂_and_distrib] at hFP₀
simp only [P₀, forall_and] at hFP₀
rcases hFP₀ with ⟨hF_sec, hF_sol, _hF_smooth, hF_A, hF_dist⟩
refine ⟨mkHtpyFormalSol F hF_sec hF_sol hFP₂, ?_, hFP₁, ?_, ?_⟩
· intro x
Expand Down Expand Up @@ -326,7 +325,7 @@ theorem RelMfld.Ample.satisfiesHPrinciple (hRample : R.Ample) (hRopen : IsOpen R
rcases inductive_htpy_construction P₀ P₁ P₂ hP₂ L.lf_φ K_cover init (𝓕₀.smooth.comp contMDiff_snd)
ind with
⟨F, hF₀, hFP₀, hFP₁, hFP₂⟩
simp only [P₀, forall₂_and_distrib] at hFP₀
simp only [P₀, forall_and] at hFP₀
rcases hFP₀ with ⟨hF_sec, hF_sol, _hF_smooth, hF_A, hF_dist⟩
refine ⟨mkHtpyFormalSol F hF_sec hF_sol hFP₂, ?_, hFP₁, ?_, ?_⟩
· intro x
Expand Down
6 changes: 0 additions & 6 deletions SphereEversion/ToMathlib/Logic/Basic.lean

This file was deleted.

0 comments on commit 62ac547

Please sign in to comment.