take into consideration whether a fact is an "intro"/"elim"/"simp" rule as an additional factor influencing the relevance filter
theory Syntax
imports Base
begin
chapter {* Concrete syntax and type-checking *}
text FIXME
section {* Parsing and printing *}
text FIXME
section {* Checking and unchecking \label{sec:term-check} *}
end