781f709bb4
We will use well-founded recursion in the definitional package
6 lines
170 B
Text
6 lines
170 B
Text
import logic.prop
|
|
|
|
inductive acc (A : Type) (R : A → A → Prop) : A → Prop :=
|
|
intro : ∀ (x : A), (∀ (y : A), R y x → acc A R y) → acc A R x
|
|
|
|
check @acc.rec
|