Skip to content

Commit

Permalink
Remove extraneous hypotheses
Browse files Browse the repository at this point in the history
  • Loading branch information
zeramorphic committed Nov 26, 2024
1 parent 214c408 commit fa12670
Showing 1 changed file with 1 addition and 2 deletions.
3 changes: 1 addition & 2 deletions ConNF/Construction/RunInduction.lean
Original file line number Diff line number Diff line change
Expand Up @@ -18,8 +18,7 @@ open Cardinal Ordinal WithBot

namespace ConNF

variable [Params.{u}] {α : Λ} (M : (β : Λ) → (β : TypeIndex) < α → Motive β)
(H : (β : Λ) → (h : (β : TypeIndex) < α) → Hypothesis (M β h) λ γ h' ↦ M γ (h'.trans h))
variable [Params.{u}]

instance : IsTrans Λ λ β γ ↦ (β : TypeIndex) < (γ : TypeIndex) :=
⟨λ _ _ _ ↦ lt_trans⟩
Expand Down

0 comments on commit fa12670

Please sign in to comment.