fix(tests): fix tests after changes is the HoTT library

This commit is contained in:
Floris van Doorn 2016-06-23 23:26:37 +01:00 committed by Leonardo de Moura
parent 17ccc283a9
commit fb81bcaeee
4 changed files with 4 additions and 3 deletions

View file

@ -5,5 +5,5 @@ definition my_elim {A P : Type} {R : A → A → Type} (Pc : A → P)
begin
induction x,
exact (Pc a),
refine (pathover_of_eq (Pp H))
refine (pathover_of_eq _ (Pp H))
end

View file

@ -4,5 +4,5 @@ definition my_elim {A P : Type} {R : A → A → Type} (Pc : A → P)
begin
induction x,
exact (Pc a),
refine (pathover_of_eq (Pp H))
refine (pathover_of_eq _ (Pp H))
end

View file

@ -27,7 +27,7 @@ section
protected definition elim {P : Type} (Pt : A → P)
(Pe : Π(a a' : A), Pt a = Pt a') (x : one_step_tr) : P :=
rec Pt (λa a', pathover_of_eq (Pe a a')) x
rec Pt (λa a', pathover_of_eq _ (Pe a a')) x
theorem rec_tr_eq {P : one_step_tr → Type} (Pt : Π(a : A), P (tr a))
(Pe : Π(a a' : A), Pt a =[tr_eq a a'] Pt a') (a a' : A)

View file

@ -1,3 +1,4 @@
open eq
set_option pp.universes true
check @homotopy.rec_on