Finish algo_metric_case
This commit is contained in:
parent
849169be7f
commit
093fc8f9cb
2 changed files with 39 additions and 5 deletions
|
@ -60,6 +60,7 @@ Fixpoint ishne {n} (a : PTm n) :=
|
|||
| VarPTm _ => true
|
||||
| PApp a _ => ishne a
|
||||
| PProj _ a => ishne a
|
||||
| PBot => true
|
||||
| _ => false
|
||||
end.
|
||||
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue