Skip to content

Commit

Permalink
Join.Core: remove unneeded universe annotations
Browse files Browse the repository at this point in the history
  • Loading branch information
jdchristensen committed Oct 24, 2023
1 parent 079d6d8 commit 3d4f109
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions theories/Homotopy/Join/Core.v
Original file line number Diff line number Diff line change
Expand Up @@ -216,8 +216,8 @@ Ltac interval_ind f a b :=

(** Similarly, for [h : JoinRecPath f g], if we have [a] and [b] and are trying to prove a goal only involving [h] and [g] evaluated at those points, we can assume that [g] is [f] and that [h] is "reflexivity". For this, we first define a lemma that is like "path induction on h", and then a tactic that uses it. *)

Definition square_ind {P : Type@{u}} (a b : P) (ab : a = b)
(Q : forall (a' b' : P) (ab' : a' = b') (ha : a = a') (hb : b = b') (k : ab @ hb = ha @ ab'), Type@{v})
Definition square_ind {P : Type} (a b : P) (ab : a = b)
(Q : forall (a' b' : P) (ab' : a' = b') (ha : a = a') (hb : b = b') (k : ab @ hb = ha @ ab'), Type)
(s : Q a b ab idpath idpath (equiv_p1_1q idpath))
: forall a' b' ab' ha hb k, Q a' b' ab' ha hb k.
Proof.
Expand Down

0 comments on commit 3d4f109

Please sign in to comment.