e499f8e20a
The new relaxed version allows us to define the "accessability" proposition and have an eliminator into Type. See justification in the new comments at inductive.cpp
6 lines
165 B
Text
6 lines
165 B
Text
import logic
|
|
|
|
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
|