fix(tests/lean/hott/433): remove bogus comment, and use rewrite tactic
Fix an issue raised by Floris. See discussion at https://github.com/leanprover/lean/issues/433
This commit is contained in:
parent
4248ad644d
commit
461c02d790
1 changed files with 2 additions and 2 deletions
|
@ -94,6 +94,7 @@ namespace pi
|
|||
definition transport_V [reducible] (P : A → Type) {x y : A} (p : x = y) (u : P y) : P x :=
|
||||
p⁻¹ ▹ u
|
||||
|
||||
open function
|
||||
protected definition functor_pi : (Π(a:A), B a) → (Π(a':A'), B' a') := (λg a', f1 a' (g (f0 a')))
|
||||
/- Equivalences -/
|
||||
definition isequiv_functor_pi [instance] (f0 : A' → A) (f1 : Π(a':A'), B (f0 a') → B' a')
|
||||
|
@ -109,8 +110,7 @@ namespace pi
|
|||
rewrite adj,
|
||||
rewrite -transport_compose,
|
||||
rewrite {f1 a' _}(ap_transport _ f1 _),
|
||||
apply (transport_V (λx, sect f0 a' ▹ x = h a') (retr (f1 _) _)),
|
||||
-- retr cannot be used as rewrite rule, the resulting type is not an equality
|
||||
rewrite (retr (f1 _) _),
|
||||
apply apD,
|
||||
intro h, beta,
|
||||
apply path_pi, intro a, esimp,
|
||||
|
|
Loading…
Reference in a new issue