You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
(F : ∀ a, (∀ a', R a' a → C a') → C a) (F' : ∀ a, (∀ a', R (f a') (f a) → C (f a')) → C (f a))
44
44
(h : ∀ a r, F (f a) r = F' a fun a' hR => r (f a') hR) (a : α') (h : WellFounded R) :
45
45
extrinsicFix (C := (C <| f ·)) (InvImage R f) F' a = extrinsicFix (C := C) R F (f a) := by
@@ -73,7 +73,7 @@ public theorem WellFounded.partialExtrinsicFix_eq [∀ a, Nonempty (C a)] (R :
73
73
apply Or.inr
74
74
refine TransGen.trans h ?_
75
75
exact .single hR⟩
76
-
have := bla (C := (C ·.val)) (R := (R ·.1 ·.1)) (f := f) (F := fun a r => F a.1fun a' hR => r ⟨a', Or.inr (by cases a.2; grind [TransGen.single]; exact .trans (.single hR) ‹_›)⟩ hR)
76
+
have := extrinsicFix_invImage (C := (C ·.val)) (R := (R ·.1 ·.1)) (f := f) (F := fun a r => F a.1fun a' hR => r ⟨a', Or.inr (by cases a.2; grind [TransGen.single]; exact .trans (.single hR) ‹_›)⟩ hR)
77
77
(F' := fun a r => F a.1fun a' hR => r ⟨a', by cases a.2; grind [TransGen.single]; exact Or.inr (.trans (.single hR) ‹_›)⟩ hR)
78
78
unfold InvImage at this
79
79
rw [this]
@@ -115,7 +115,7 @@ public theorem WellFounded.partialExtrinsicFix₂_eq_partialExtrinsicFix [∀ a
115
115
simp only [partialExtrinsicFix, partialExtrinsicFix₂, extrinsicFix₂]
116
116
let f (x : ((a' : α) ×' { b' // PSigma.mk a' b' = ⟨a, b⟩ ∨ TransGen R ⟨a', b'⟩ ⟨a, b⟩ })) : { a' // a' = ⟨a, b⟩ ∨ TransGen R a' ⟨a, b⟩ } :=
117
117
⟨⟨x.1, x.2.1⟩, x.2.2⟩
118
-
have := bla (C := fun a => C₂ a.1.1 a.1.2) (f := f) (R := (R ·.1 ·.1))
118
+
have := extrinsicFix_invImage (C := fun a => C₂ a.1.1 a.1.2) (f := f) (R := (R ·.1 ·.1))
119
119
(F := fun a r => F a.1.1 a.1.2fun a' b' hR => r ⟨⟨a', b'⟩, ?refine_a⟩ hR)
120
120
(F' := fun a r => F a.1 a.2.1fun a' b' hR => r ⟨a', b', ?refine_b⟩ hR)
0 commit comments